Skip to content

Commit

Permalink
Update Tutorial_Chaining_Tactics.v
Browse files Browse the repository at this point in the history
  • Loading branch information
thomas-lamiaux authored Nov 2, 2024
1 parent e967e25 commit 0d3ab6e
Showing 1 changed file with 2 additions and 4 deletions.
6 changes: 2 additions & 4 deletions src/Tutorial_Chaining_Tactics.v
Original file line number Diff line number Diff line change
Expand Up @@ -38,9 +38,7 @@
*)

Require Import Lia.

Section Chaining.
Section Chaining.
Context (A B C D E F : Type).

Set Printing Parentheses.
Expand Down Expand Up @@ -539,4 +537,4 @@ Goal A -> B -> C -> D -> E -> F.
Fail do 8 intros ?.
Abort.

End Chaining.
End Chaining.

0 comments on commit 0d3ab6e

Please sign in to comment.