Skip to content

Commit 96175ed

Browse files
committed
refactoring; remove explicit definition of CounterExample
1 parent fb8480b commit 96175ed

File tree

1 file changed

+5
-8
lines changed

1 file changed

+5
-8
lines changed

src/Induction/NoInfiniteDescent.agda

Lines changed: 5 additions & 8 deletions
Original file line numberDiff line numberDiff line change
@@ -14,13 +14,15 @@ open import Data.Nat.Base as ℕ using (ℕ; zero; suc)
1414
open import Data.Nat.Properties as ℕ
1515
open import Data.Product.Base using (_,_; proj₁; ∃-syntax; _×_)
1616
open import Function.Base using (_∘_)
17-
open import Induction.WellFounded using (WellFounded; Acc; acc; acc-inverse; module Some)
17+
open import Induction.WellFounded
18+
using (WellFounded; Acc; acc; acc-inverse; module Some)
1819
open import Level using (Level)
1920
open import Relation.Binary.Core using (Rel)
2021
open import Relation.Binary.Construct.Closure.Transitive
2122
open import Relation.Binary.PropositionalEquality.Core
2223
open import Relation.Nullary.Negation.Core as Negation using (¬_)
23-
open import Relation.Unary using (Pred; _∩_; _⇒_; Universal; IUniversal; Stable)
24+
open import Relation.Unary
25+
using (Pred; ∁; _∩_; _⇒_; Universal; IUniversal; Stable)
2426

2527
private
2628
variable
@@ -199,14 +201,9 @@ module FurtherCorollaries {_<_ : Rel A r} (P : Pred A ℓ) where
199201
------------------------------------------------------------------------
200202
-- Finally: the (classical) 'no smallest counterexample' principle itself
201203

202-
-- these belong in Relation.Unary
203-
204-
CounterExample : Pred A ℓ Pred A ℓ
205-
CounterExample P = ¬_ ∘ P
206-
207204
module _ {_<_ : Rel A r} {P : Pred A ℓ} (stable : Stable P) where
208205

209-
open FurtherCorollaries {_<_ = _<_} (CounterExample P)
206+
open FurtherCorollaries {_<_ = _<_} ( P)
210207
using (acc⇒noInfiniteDescent⁺; wf⇒noInfiniteDescent⁺)
211208
renaming (Acc⇒Descent⁺ to NoSmallestCounterExample)
212209

0 commit comments

Comments
 (0)