Skip to content

Commit

Permalink
Adapt to split_stdlib
Browse files Browse the repository at this point in the history
  • Loading branch information
proux01 committed Jul 22, 2024
1 parent 9ba18c4 commit 1d55d08
Show file tree
Hide file tree
Showing 3 changed files with 3 additions and 3 deletions.
2 changes: 1 addition & 1 deletion src/Classes.v
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
From Coq Require Import List Morphisms Recdef ZArith ZArith.Znat Arith.
From Coq Require Import List Morphisms Recdef ZArith Znat Arith.
From QuickChick Require Import Sets Tactics Producer Generators Enumerators.

Set Bullet Behavior "Strict Subproofs".
Expand Down
2 changes: 1 addition & 1 deletion src/LazyList.v
Original file line number Diff line number Diff line change
Expand Up @@ -344,7 +344,7 @@ Fixpoint filter_LazyList {A} (p : A -> bool) (l : LazyList A) :=
else filter_LazyList p (t tt)
end.

Require Import Coq.Logic.ClassicalFacts.
From Coq.Logic Require Import ClassicalFacts.

Axiom EM : excluded_middle.

Expand Down
2 changes: 1 addition & 1 deletion src/TacticsUtil.v.cppo
Original file line number Diff line number Diff line change
Expand Up @@ -27,7 +27,7 @@ Ltac2 Notation "inv" h(ident) := inv_tac h.
Local Ltac2 exfalso_tac () := ltac1:(exfalso).
Ltac2 Notation "exfalso" := exfalso_tac ().

Local Ltac2 lia_ltac1 () := ltac1:(micromega.Lia.lia).
Local Ltac2 lia_ltac1 () := ltac1:(Lia.lia).
Ltac2 Notation "lia" := lia_ltac1 ().

Ltac2 inv := fun (h : ident) => inversion h; subst.
Expand Down

0 comments on commit 1d55d08

Please sign in to comment.