Skip to content

Commit

Permalink
Merge pull request #18 from coq-community/ignore-warnings
Browse files Browse the repository at this point in the history
Ignore warnings in 8.12
  • Loading branch information
chdoc authored Oct 5, 2020
2 parents 39b75d2 + 88906cd commit 62ad0b7
Show file tree
Hide file tree
Showing 3 changed files with 4 additions and 2 deletions.
2 changes: 2 additions & 0 deletions _CoqProject
Original file line number Diff line number Diff line change
@@ -1,6 +1,8 @@
-Q theories RegLang
-arg -w -arg -notation-overridden
-arg -w -arg -duplicate-clear
-arg -w -arg -notation-incompatible-format
-arg -w -arg -omega-is-deprecated
theories/misc.v
theories/setoid_leq.v
theories/languages.v
Expand Down
2 changes: 1 addition & 1 deletion theories/dune
Original file line number Diff line number Diff line change
Expand Up @@ -2,4 +2,4 @@
(name RegLang)
(package coq-reglang)
(synopsis "Representations of regular languages (i.e., regexps, various types of automata, and WS1S) with equivalence proofs, in Coq and MathComp")
(flags -w -notation-overridden -w -duplicate-clear))
(flags -w -notation-overridden -w -duplicate-clear -w -notation-incompatible-format -w -omega-is-deprecated))
2 changes: 1 addition & 1 deletion theories/misc.v
Original file line number Diff line number Diff line change
Expand Up @@ -28,7 +28,7 @@ Lemma eqb_iff (b1 b2 : bool) : (b1 <-> b2) <-> (b1 = b2).
Proof. split => [[A B]|->//]. exact/idP/idP. Qed.

(* equivalence of type inhabitation *)
CoInductive iffT T1 T2 := IffT of (T1 -> T2) & (T2 -> T1).
Variant iffT T1 T2 := IffT of (T1 -> T2) & (T2 -> T1).
Notation "T1 <-T-> T2" := (iffT T1 T2) (at level 30).

Definition iffT_LR T1 T2 : iffT T1 T2 -> T1 -> T2. by case. Qed.
Expand Down

0 comments on commit 62ad0b7

Please sign in to comment.