2014-12-23 20:35:06 +00:00
|
|
|
/-
|
|
|
|
Copyright (c) 2014 Microsoft Corporation. All rights reserved.
|
|
|
|
Released under Apache 2.0 license as described in the file LICENSE.
|
|
|
|
|
|
|
|
Module: data.string
|
|
|
|
Author: Leonardo de Moura
|
|
|
|
-/
|
2014-12-01 04:34:12 +00:00
|
|
|
import data.bool
|
2015-01-10 22:07:20 +00:00
|
|
|
open bool
|
2014-07-02 15:36:05 +00:00
|
|
|
|
2015-01-10 22:07:20 +00:00
|
|
|
protected definition char.is_inhabited [instance] : inhabited char :=
|
|
|
|
inhabited.mk (char.mk ff ff ff ff ff ff ff ff)
|
2014-07-04 21:25:44 +00:00
|
|
|
|
2015-01-10 22:07:20 +00:00
|
|
|
protected definition string.is_inhabited [instance] : inhabited string :=
|
|
|
|
inhabited.mk string.empty
|
2015-05-04 03:46:33 +00:00
|
|
|
|
|
|
|
open decidable
|
|
|
|
|
|
|
|
definition decidable_eq_char [instance] : ∀ c₁ c₂ : char, decidable (c₁ = c₂) :=
|
|
|
|
begin
|
|
|
|
intro c₁ c₂,
|
|
|
|
cases c₁ with a₁ a₂ a₃ a₄ a₅ a₆ a₇ a₈,
|
|
|
|
cases c₂ with b₁ b₂ b₃ b₄ b₅ b₆ b₇ b₈,
|
|
|
|
apply (@by_cases (a₁ = b₁)), intros,
|
|
|
|
apply (@by_cases (a₂ = b₂)), intros,
|
|
|
|
apply (@by_cases (a₃ = b₃)), intros,
|
|
|
|
apply (@by_cases (a₄ = b₄)), intros,
|
|
|
|
apply (@by_cases (a₅ = b₅)), intros,
|
|
|
|
apply (@by_cases (a₆ = b₆)), intros,
|
|
|
|
apply (@by_cases (a₇ = b₇)), intros,
|
|
|
|
apply (@by_cases (a₈ = b₈)), intros,
|
|
|
|
left, congruence, repeat assumption,
|
|
|
|
repeat (intro n; right; intro h; injection h; refine absurd _ n; assumption)
|
|
|
|
end
|
|
|
|
|
|
|
|
open string
|
|
|
|
|
|
|
|
definition decidable_eq_string [instance] : ∀ s₁ s₂ : string, decidable (s₁ = s₂)
|
|
|
|
| empty empty := by left; reflexivity
|
|
|
|
| empty (str c₂ r₂) := by right; contradiction
|
|
|
|
| (str c₁ r₁) empty := by right; contradiction
|
|
|
|
| (str c₁ r₁) (str c₂ r₂) :=
|
|
|
|
match decidable_eq_char c₁ c₂ with
|
|
|
|
| inl e₁ :=
|
|
|
|
match decidable_eq_string r₁ r₂ with
|
|
|
|
| inl e₂ := by left; congruence; repeat assumption
|
|
|
|
| inr n₂ := by right; intro h; injection h; refine absurd _ n₂; assumption
|
|
|
|
end
|
|
|
|
| inr n₁ := by right; intro h; injection h; refine absurd _ n₁; assumption
|
|
|
|
end
|