refactor(library/init/{funext,quot}.lean): adjust comments and headers

This commit is contained in:
Jeremy Avigad 2015-04-05 10:11:53 -04:00
parent 6596217a84
commit 74ff43a543
2 changed files with 5 additions and 4 deletions

View file

@ -2,21 +2,21 @@
Copyright (c) 2015 Microsoft Corporation. All rights reserved. Copyright (c) 2015 Microsoft Corporation. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE. Released under Apache 2.0 license as described in the file LICENSE.
Module: init.funext
Author: Jeremy Avigad Author: Jeremy Avigad
function extensionality from quotients Function extensionality follows from quotients.
-/ -/
prelude prelude
import init.quot init.logic import init.quot init.logic
/- function extensionality follows from quotients -/
section section
open quot open quot
variables {A : Type} {B : A → Type} variables {A : Type} {B : A → Type}
private definition fun_eqv (f₁ f₂ : Πx : A, B x) : Prop := ∀x, f₁ x = f₂ x private definition fun_eqv (f₁ f₂ : Πx : A, B x) : Prop := ∀x, f₁ x = f₂ x
infix `~` := fun_eqv -- this is "~" infix `~` := fun_eqv
private theorem fun_eqv.refl (f : Πx : A, B x) : f ~ f := take x, rfl private theorem fun_eqv.refl (f : Πx : A, B x) : f ~ f := take x, rfl

View file

@ -2,9 +2,10 @@
Copyright (c) 2015 Microsoft Corporation. All rights reserved. Copyright (c) 2015 Microsoft Corporation. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE. Released under Apache 2.0 license as described in the file LICENSE.
Module: init.quot
Author: Leonardo de Moura Author: Leonardo de Moura
Quotient types Quotient types.
-/ -/
prelude prelude
import init.sigma init.setoid init.logic import init.sigma init.setoid init.logic