Search is not available for this dataset
text
string | meta
dict |
---|---|
module Structure.Operator.Proofs.Util where
import Lvl
open import Data
open import Data.Tuple
open import Functional hiding (id)
open import Function.Equals
import Function.Names as Names
import Lang.Vars.Structure.Operator
open Lang.Vars.Structure.Operator.Select
open import Logic.IntroInstances
open import Logic.Predicate
open import Structure.Setoid
open import Structure.Function.Domain
import Structure.Operator.Names as Names
open import Structure.Operator.Properties
open import Structure.Operator
open import Structure.Relator.Properties
open import Syntax.Transitivity
open import Type
module One {ℓ ℓₑ} {T : Type{ℓ}} ⦃ equiv : Equiv{ℓₑ}(T) ⦄ {_▫_ : T → T → T} where
open Lang.Vars.Structure.Operator.One ⦃ equiv = equiv ⦄ {_▫_ = _▫_}
-- TODO: Rename this to associate-commute4-commuting
associate-commute4 : let _ = op , assoc in ∀{a b c d} → Names.Commuting(_▫_)(b)(c) → ((a ▫ b) ▫ (c ▫ d) ≡ (a ▫ c) ▫ (b ▫ d))
associate-commute4 {a}{b}{c}{d} com =
(a ▫ b) ▫ (c ▫ d) 🝖-[ symmetry(_≡_) (associativity(_▫_) {a ▫ b} {c} {d}) ]
((a ▫ b) ▫ c) ▫ d 🝖-[ congruence₂ₗ(_▫_)(d) (associativity(_▫_) {a} {b} {c}) ]
(a ▫ (b ▫ c)) ▫ d 🝖-[ (congruence₂ₗ(_▫_)(d) ∘ congruence₂ᵣ(_▫_)(a)) com ]
(a ▫ (c ▫ b)) ▫ d 🝖-[ associativity(_▫_) {a} {c ▫ b} {d} ]
a ▫ ((c ▫ b) ▫ d) 🝖-[ congruence₂ᵣ(_▫_)(a) (associativity(_▫_) {c} {b} {d}) ]
a ▫ (c ▫ (b ▫ d)) 🝖-[ symmetry(_≡_) (associativity(_▫_) {a} {c} {b ▫ d}) ]
(a ▫ c) ▫ (b ▫ d) 🝖-end
-- TODO: Rename this to associate-commute4
associate-commute4-c : let _ = op , assoc , comm in ∀{a b c d} → ((a ▫ b) ▫ (c ▫ d) ≡ (a ▫ c) ▫ (b ▫ d))
associate-commute4-c = associate-commute4(commutativity(_▫_))
associate4-123-321 : let _ = op , assoc in ∀{a b c d} → (((a ▫ b) ▫ c) ▫ d ≡ a ▫ (b ▫ (c ▫ d)))
associate4-123-321 {a}{b}{c}{d} = associativity(_▫_) 🝖 associativity(_▫_)
associate4-123-213 : let _ = op , assoc in ∀{a b c d} → (((a ▫ b) ▫ c) ▫ d ≡ (a ▫ (b ▫ c)) ▫ d)
associate4-123-213 {a}{b}{c}{d} = congruence₂ₗ(_▫_)(_) (associativity(_▫_))
associate4-321-231 : let _ = op , assoc in ∀{a b c d} → (a ▫ (b ▫ (c ▫ d)) ≡ a ▫ ((b ▫ c) ▫ d))
associate4-321-231 {a}{b}{c}{d} = congruence₂ᵣ(_▫_)(_) (symmetry(_≡_) (associativity(_▫_)))
associate4-231-222 : let _ = op , assoc in ∀{a b c d} → (a ▫ ((b ▫ c) ▫ d) ≡ (a ▫ b) ▫ (c ▫ d))
associate4-231-222 {a}{b}{c}{d} = symmetry(_≡_) associate4-321-231 🝖 symmetry(_≡_) associate4-123-321 🝖 associativity(_▫_)
associate4-213-222 : let _ = op , assoc in ∀{a b c d} → ((a ▫ (b ▫ c)) ▫ d ≡ (a ▫ b) ▫ (c ▫ d))
associate4-213-222 {a}{b}{c}{d} = associativity(_▫_) 🝖 associate4-231-222
commuteᵣ-assocₗ : let _ = op , assoc , comm in ∀{a b c} → (((a ▫ b) ▫ c) ≡ ((a ▫ c) ▫ b))
commuteᵣ-assocₗ {a}{b}{c} =
(a ▫ b) ▫ c 🝖-[ associativity(_▫_) ]
a ▫ (b ▫ c) 🝖-[ congruence₂ᵣ(_▫_)(_) (commutativity(_▫_)) ]
a ▫ (c ▫ b) 🝖-[ associativity(_▫_) ]-sym
(a ▫ c) ▫ b 🝖-end
commuteₗ-assocᵣ : let _ = op , assoc , comm in ∀{a b c} → ((a ▫ (b ▫ c)) ≡ (b ▫ (a ▫ c)))
commuteₗ-assocᵣ {a}{b}{c} =
a ▫ (b ▫ c) 🝖-[ associativity(_▫_) ]-sym
(a ▫ b) ▫ c 🝖-[ congruence₂ₗ(_▫_)(_) (commutativity(_▫_)) ]
(b ▫ a) ▫ c 🝖-[ associativity(_▫_) ]
b ▫ (a ▫ c) 🝖-end
commuteᵣ-assocᵣ : let _ = op , assoc , comm in ∀{a b c} → ((a ▫ (b ▫ c)) ≡ ((a ▫ c) ▫ b))
commuteᵣ-assocᵣ = symmetry(_≡_) (associativity(_▫_)) 🝖 commuteᵣ-assocₗ
-- TODO: Rename and generalize this (See commuteBoth in Structure.Operator.Properties)
commuteBothTemp : let _ = comm in ∀{a₁ a₂ b₁ b₂} → (a₁ ▫ a₂ ≡ b₁ ▫ b₂) → (a₂ ▫ a₁ ≡ b₂ ▫ b₁)
commuteBothTemp {a₁} {a₂} {b₁} {b₂} p =
a₂ ▫ a₁ 🝖-[ commutativity(_▫_) ]-sym
a₁ ▫ a₂ 🝖-[ p ]
b₁ ▫ b₂ 🝖-[ commutativity(_▫_) ]
b₂ ▫ b₁ 🝖-end
moveₗ-to-inv : let _ = op , assoc , select-invₗ(idₗ)(identₗ)(invₗ)(inverₗ) in ∀{a b c} → (a ▫ b ≡ c) → (b ≡ invₗ(a) ▫ c)
moveₗ-to-inv {idₗ = idₗ} {invₗ = invₗ} {a = a} {b} {c} abc =
b 🝖-[ identityₗ(_▫_)(idₗ) ]-sym
idₗ ▫ b 🝖-[ congruence₂ₗ(_▫_)(b) (inverseFunctionₗ(_▫_)(invₗ)) ]-sym
(invₗ a ▫ a) ▫ b 🝖-[ associativity(_▫_) ]
invₗ a ▫ (a ▫ b) 🝖-[ congruence₂ᵣ(_▫_)(invₗ a) abc ]
invₗ a ▫ c 🝖-end
moveᵣ-to-inv : let _ = op , assoc , select-invᵣ(idᵣ)(identᵣ)(invᵣ)(inverᵣ) in ∀{a b c} → (a ▫ b ≡ c) → (a ≡ c ▫ invᵣ(b))
moveᵣ-to-inv {idᵣ = idᵣ} {invᵣ = invᵣ} {a = a} {b} {c} abc =
a 🝖-[ identityᵣ(_▫_)(idᵣ) ]-sym
a ▫ idᵣ 🝖-[ congruence₂ᵣ(_▫_)(a) (inverseFunctionᵣ(_▫_)(invᵣ)) ]-sym
a ▫ (b ▫ invᵣ b) 🝖-[ associativity(_▫_) ]-sym
(a ▫ b) ▫ invᵣ b 🝖-[ congruence₂ₗ(_▫_)(invᵣ b) abc ]
c ▫ invᵣ b 🝖-end
moveₗ-from-inv : let _ = op , assoc , select-idₗ(id)(identₗ) , select-invᵣ(id)(identᵣ)(invᵣ)(inverᵣ) in ∀{a b c} → (a ▫ b ≡ c) ← (b ≡ invᵣ(a) ▫ c)
moveₗ-from-inv {id = id} {invᵣ = invᵣ} {a = a} {b} {c} bac =
a ▫ b 🝖-[ congruence₂ᵣ(_▫_)(a) bac ]
a ▫ (invᵣ a ▫ c) 🝖-[ associativity(_▫_) ]-sym
(a ▫ invᵣ a) ▫ c 🝖-[ congruence₂ₗ(_▫_)(c) (inverseFunctionᵣ(_▫_)(invᵣ)) ]
id ▫ c 🝖-[ identityₗ(_▫_)(id) ]
c 🝖-end
moveᵣ-from-inv : let _ = op , assoc , select-idᵣ(id)(identᵣ) , select-invₗ(id)(identₗ)(invₗ)(inverₗ) in ∀{a b c} → (a ▫ b ≡ c) ← (a ≡ c ▫ invₗ(b))
moveᵣ-from-inv {id = id} {invₗ = invₗ} {a = a} {b} {c} acb =
a ▫ b 🝖-[ congruence₂ₗ(_▫_)(b) acb ]
(c ▫ invₗ b) ▫ b 🝖-[ associativity(_▫_) ]
c ▫ (invₗ b ▫ b) 🝖-[ congruence₂ᵣ(_▫_)(c) (inverseFunctionₗ(_▫_)(invₗ)) ]
c ▫ id 🝖-[ identityᵣ(_▫_)(id) ]
c 🝖-end
module OneTypeTwoOp {ℓ ℓₑ} {T : Type{ℓ}} ⦃ equiv : Equiv{ℓₑ}(T) ⦄ {_▫₁_ _▫₂_ : T → T → T} where
open Lang.Vars.Structure.Operator.OneTypeTwoOp ⦃ equiv = equiv ⦄ {_▫₁_ = _▫₁_} {_▫₂_ = _▫₂_}
cross-distribute : let _ = op₂ , distriₗ , distriᵣ in ∀{a b c d} → (a ▫₂ b) ▫₁ (c ▫₂ d) ≡ ((a ▫₁ c) ▫₂ (b ▫₁ c)) ▫₂ ((a ▫₁ d) ▫₂ (b ▫₁ d))
cross-distribute {a = a}{b}{c}{d} =
(a ▫₂ b) ▫₁ (c ▫₂ d) 🝖-[ distributivityₗ(_▫₁_)(_▫₂_) ]
((a ▫₂ b) ▫₁ c) ▫₂ ((a ▫₂ b) ▫₁ d) 🝖-[ congruence₂(_▫₂_) (distributivityᵣ(_▫₁_)(_▫₂_)) (distributivityᵣ(_▫₁_)(_▫₂_)) ]
((a ▫₁ c) ▫₂ (b ▫₁ c)) ▫₂ ((a ▫₁ d) ▫₂ (b ▫₁ d)) 🝖-end
moveₗ-to-invOp : let _ = op₂ , inverOpₗ in ∀{a b c} → (a ▫₁ b ≡ c) → (b ≡ a ▫₂ c)
moveₗ-to-invOp {a = a} {b} {c} abc =
b 🝖[ _≡_ ]-[ inverseOperₗ(_▫₁_)(_▫₂_) ]-sym
a ▫₂ (a ▫₁ b) 🝖[ _≡_ ]-[ congruence₂ᵣ(_▫₂_)(a) abc ]
a ▫₂ c 🝖-end
moveᵣ-to-invOp : let _ = op₂ , inverOpᵣ in ∀{a b c} → (a ▫₁ b ≡ c) → (a ≡ c ▫₂ b)
moveᵣ-to-invOp {a = a} {b} {c} abc =
a 🝖[ _≡_ ]-[ inverseOperᵣ(_▫₁_)(_▫₂_) ]-sym
(a ▫₁ b) ▫₂ b 🝖[ _≡_ ]-[ congruence₂ₗ(_▫₂_)(b) abc ]
c ▫₂ b 🝖-end
| {
"alphanum_fraction": 0.5248373743,
"avg_line_length": 51.2424242424,
"ext": "agda",
"hexsha": "3da926bccdd5fa6bde402ced10159bffa504d189",
"lang": "Agda",
"max_forks_count": null,
"max_forks_repo_forks_event_max_datetime": null,
"max_forks_repo_forks_event_min_datetime": null,
"max_forks_repo_head_hexsha": "70f4fba849f2fd779c5aaa5af122ccb6a5b271ba",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "Lolirofle/stuff-in-agda",
"max_forks_repo_path": "Structure/Operator/Proofs/Util.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "70f4fba849f2fd779c5aaa5af122ccb6a5b271ba",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "Lolirofle/stuff-in-agda",
"max_issues_repo_path": "Structure/Operator/Proofs/Util.agda",
"max_line_length": 148,
"max_stars_count": 6,
"max_stars_repo_head_hexsha": "70f4fba849f2fd779c5aaa5af122ccb6a5b271ba",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "Lolirofle/stuff-in-agda",
"max_stars_repo_path": "Structure/Operator/Proofs/Util.agda",
"max_stars_repo_stars_event_max_datetime": "2022-02-05T06:53:22.000Z",
"max_stars_repo_stars_event_min_datetime": "2020-04-07T17:58:13.000Z",
"num_tokens": 3372,
"size": 6764
} |
-- {-# OPTIONS -v tc.size:100 #-}
module SizedTypesMergeSort where
open import Common.Size
open import Common.Prelude using (Bool; true; false; if_then_else_)
open import Common.Product
module Old where
-- sized lists
data List (A : Set) : {_ : Size} -> Set where
[] : {size : Size} -> List A {↑ size}
_::_ : {size : Size} -> A -> List A {size} -> List A {↑ size}
-- CPS split (non-size increasing)
split : {A : Set}{i : Size} -> List A {i} ->
{C : Set} -> (List A {i} -> List A {i} -> C) -> C
split [] k = k [] []
split (x :: xs) k = split xs (\ l r -> k (x :: r) l)
module Sort (A : Set) (compare : A -> A -> {B : Set} -> B -> B -> B) where
-- Andreas, 4 Sep 2008
-- the size indices i and j should not be necessary here
-- but without them, the termination checker does not recognise that
-- the pattern x :: xs is equal to the term x :: xs
-- I suspect that _::_ {∞} x xs is not equal to itself since ∞ is a term
-- not a constructor or variable
merge : {i j : Size} -> List A {i} -> List A {j} -> List A
merge [] ys = ys
merge xs [] = xs
merge (x :: xs) (y :: ys) =
compare x y (x :: merge xs (y :: ys))
(y :: merge (x :: xs) ys)
sort : {i : Size} -> List A {i} -> List A
sort [] = []
sort (x :: []) = x :: []
sort (x :: (y :: xs)) = split xs (\ l r -> merge (sort (x :: l))
(sort (y :: r)))
module New where
-- sized lists
data List A {i} : Set where
[] : List A
_::_ : {i' : Size< i} → A → List A {i'} → List A
module CPS where
-- CPS split (non-size increasing)
split : ∀ {A i} → List A {i} →
{C : Set} → (List A {i} → List A {i} → C) → C
split [] k = k [] []
split (x :: xs) k = split xs (\ l r → k (x :: r) l)
module Sort (A : Set) (compare : A → A → {B : Set} → B → B → B) where
merge : List A → List A → List A
merge [] ys = ys
merge xs [] = xs
merge (x :: xs) (y :: ys) =
compare x y (x :: merge xs (y :: ys))
(y :: merge (x :: xs) ys)
sort : {i : Size} → List A {i} → List A
sort [] = []
sort (x :: []) = x :: []
sort (x :: (y :: xs)) = split xs (\ l r → merge (sort (x :: l))
(sort (y :: r)))
module Direct where
split : ∀ {A i} → List A {i} → List A {i} × List A {i}
split [] = [] , []
split (x :: xs) = let l , r = split xs in (x :: r) , l
module Sort (A : Set) (_≤_ : A → A → Bool) where
merge : List A → List A → List A
merge [] ys = ys
merge xs [] = xs
merge (x :: xs) (y :: ys) =
if x ≤ y then (x :: merge xs (y :: ys))
else (y :: merge (x :: xs) ys)
sort : {i : Size} → List A {i} → List A
sort [] = []
sort (x :: []) = x :: []
sort (x :: (y :: xs)) = let l , r = split xs in merge (sort (x :: l))
(sort (y :: r))
| {
"alphanum_fraction": 0.4263292761,
"avg_line_length": 31.22,
"ext": "agda",
"hexsha": "1f9a904db5df2a1d8b6c5f0c63cb912de1e089f4",
"lang": "Agda",
"max_forks_count": 1,
"max_forks_repo_forks_event_max_datetime": "2019-03-05T20:02:38.000Z",
"max_forks_repo_forks_event_min_datetime": "2019-03-05T20:02:38.000Z",
"max_forks_repo_head_hexsha": "c0ae7d20728b15d7da4efff6ffadae6fe4590016",
"max_forks_repo_licenses": [
"BSD-3-Clause"
],
"max_forks_repo_name": "redfish64/autonomic-agda",
"max_forks_repo_path": "test/Succeed/SizedTypesMergeSort.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "c0ae7d20728b15d7da4efff6ffadae6fe4590016",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"BSD-3-Clause"
],
"max_issues_repo_name": "redfish64/autonomic-agda",
"max_issues_repo_path": "test/Succeed/SizedTypesMergeSort.agda",
"max_line_length": 76,
"max_stars_count": 3,
"max_stars_repo_head_hexsha": "c0ae7d20728b15d7da4efff6ffadae6fe4590016",
"max_stars_repo_licenses": [
"BSD-3-Clause"
],
"max_stars_repo_name": "redfish64/autonomic-agda",
"max_stars_repo_path": "test/Succeed/SizedTypesMergeSort.agda",
"max_stars_repo_stars_event_max_datetime": "2015-12-07T20:14:00.000Z",
"max_stars_repo_stars_event_min_datetime": "2015-03-28T14:51:03.000Z",
"num_tokens": 979,
"size": 3122
} |
------------------------------------------------------------------------
-- A formalisation of one variant of the language χ, along with a
-- number of properties
--
-- Nils Anders Danielsson
------------------------------------------------------------------------
-- A description of the language χ, as well as some of the definitions
-- and proofs used in this development, can be found in "The language
-- χ" by Bengt Nordström (edited by me):
--
-- * https://chalmers.instructure.com/courses/10744/file_contents/course%20files/reading/The_language_chi.pdf
--
-- See also the following lecture slides:
--
-- * https://chalmers.instructure.com/courses/10744/file_contents/course%20files/lectures/L4.pdf
-- * https://chalmers.instructure.com/courses/10744/file_contents/course%20files/lectures/L5.pdf
-- * https://chalmers.instructure.com/courses/10744/file_contents/course%20files/lectures/L6.pdf
module README where
-- Atoms.
import Atom
-- Various constants.
import Constants
-- A specification of the language χ.
import Chi
-- The semantics is deterministic.
import Deterministic
-- Values.
import Values
-- Some cancellation lemmas.
import Cancellation
-- "Reasoning" combinators.
import Reasoning
-- The abstract syntax is a set, and the semantics is propositional.
import Propositional
-- The "terminates" relation.
import Termination
-- Compatibility lemmas.
import Compatibility
-- Some substitution lemmas.
import Substitution
-- Definitions of "free in" and "closed", along with some properties.
import Free-variables
-- Alpha-equivalence.
import Alpha-equivalence
-- Encoders and decoders.
import Coding
-- Encoder and decoder instances.
import Coding.Instances
-- Encoder and decoder instances for Atom.χ-ℕ-atoms.
import Coding.Instances.Nat
-- Internal coding.
import Internal-coding
-- Some χ program combinators.
import Combinators
-- The rec construction can be encoded using λ-terms.
import Recursion-without-rec
-- Definition of the size of an expression, along with some
-- properties.
import Expression-size
-- A self-interpreter (without correctness proof).
import Self-interpreter
-- Partial functions, computability.
import Computability
-- The halting problem.
import Halting-problem
-- Rice's theorem.
import Rices-theorem
-- A theorem related to pointwise equality.
import Pointwise-equality
| {
"alphanum_fraction": 0.718381113,
"avg_line_length": 19.4426229508,
"ext": "agda",
"hexsha": "9491fbbb6f14691e259259c17e04a9dd902a8d34",
"lang": "Agda",
"max_forks_count": null,
"max_forks_repo_forks_event_max_datetime": null,
"max_forks_repo_forks_event_min_datetime": null,
"max_forks_repo_head_hexsha": "30966769b8cbd46aa490b6964a4aa0e67a7f9ab1",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "nad/chi",
"max_forks_repo_path": "README.agda",
"max_issues_count": 1,
"max_issues_repo_head_hexsha": "30966769b8cbd46aa490b6964a4aa0e67a7f9ab1",
"max_issues_repo_issues_event_max_datetime": "2020-06-08T11:08:25.000Z",
"max_issues_repo_issues_event_min_datetime": "2020-05-21T23:29:54.000Z",
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "nad/chi",
"max_issues_repo_path": "README.agda",
"max_line_length": 109,
"max_stars_count": 2,
"max_stars_repo_head_hexsha": "30966769b8cbd46aa490b6964a4aa0e67a7f9ab1",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "nad/chi",
"max_stars_repo_path": "README.agda",
"max_stars_repo_stars_event_max_datetime": "2020-10-20T16:27:00.000Z",
"max_stars_repo_stars_event_min_datetime": "2020-05-21T22:58:07.000Z",
"num_tokens": 521,
"size": 2372
} |
open import MLib.Algebra.PropertyCode
open import MLib.Algebra.PropertyCode.Structures
module MLib.Matrix.SemiTensor {c ℓ} (struct : Struct bimonoidCode c ℓ) where
open import MLib.Matrix.SemiTensor.Core struct using (_⋉_) public
open import MLib.Matrix.SemiTensor.GeneralizesMul struct public
| {
"alphanum_fraction": 0.8243243243,
"avg_line_length": 37,
"ext": "agda",
"hexsha": "7faef95b2482ca717b14da14b24aa22d893bb2d7",
"lang": "Agda",
"max_forks_count": null,
"max_forks_repo_forks_event_max_datetime": null,
"max_forks_repo_forks_event_min_datetime": null,
"max_forks_repo_head_hexsha": "e26ae2e0aa7721cb89865aae78625a2f3fd2b574",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "bch29/agda-matrices",
"max_forks_repo_path": "src/MLib/Matrix/SemiTensor.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "e26ae2e0aa7721cb89865aae78625a2f3fd2b574",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "bch29/agda-matrices",
"max_issues_repo_path": "src/MLib/Matrix/SemiTensor.agda",
"max_line_length": 76,
"max_stars_count": null,
"max_stars_repo_head_hexsha": "e26ae2e0aa7721cb89865aae78625a2f3fd2b574",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "bch29/agda-matrices",
"max_stars_repo_path": "src/MLib/Matrix/SemiTensor.agda",
"max_stars_repo_stars_event_max_datetime": null,
"max_stars_repo_stars_event_min_datetime": null,
"num_tokens": 78,
"size": 296
} |
{-# OPTIONS --without-K --safe #-}
module Categories.Category.Instance.Monoidals where
open import Level
open import Categories.Category
open import Categories.Category.Helper
open import Categories.Category.Monoidal
open import Categories.Functor.Monoidal
open import Categories.Functor.Monoidal.Properties
open import Categories.NaturalTransformation.NaturalIsomorphism.Monoidal
module _ o ℓ e where
Monoidals : Category (suc (o ⊔ ℓ ⊔ e)) (o ⊔ ℓ ⊔ e) (o ⊔ ℓ ⊔ e)
Monoidals = categoryHelper record
{ Obj = MonoidalCategory o ℓ e
; _⇒_ = MonoidalFunctor
; _≈_ = Lax._≃_
; id = idF-Monoidal _
; _∘_ = ∘-Monoidal
-- NOTE: these η-expanded versions typecheck much faster...
; assoc = λ {_ _ _ _ F G H} → associator {F = F} {G} {H}
; identityˡ = λ {_ _ F} → unitorˡ {F = F}
; identityʳ = λ {_ _ F} → unitorʳ {F = F}
; equiv = isEquivalence
; ∘-resp-≈ = _ⓘₕ_
}
where open Lax
StrongMonoidals : Category (suc (o ⊔ ℓ ⊔ e)) (o ⊔ ℓ ⊔ e) (o ⊔ ℓ ⊔ e)
StrongMonoidals = categoryHelper record
{ Obj = MonoidalCategory o ℓ e
; _⇒_ = StrongMonoidalFunctor
; _≈_ = Strong._≃_
; id = idF-StrongMonoidal _
; _∘_ = ∘-StrongMonoidal
-- NOTE: these η-expanded versions typecheck much faster...
; assoc = λ {_ _ _ _ F G H} → associator {F = F} {G} {H}
; identityˡ = λ {_ _ F} → unitorˡ {F = F}
; identityʳ = λ {_ _ F} → unitorʳ {F = F}
; equiv = isEquivalence
; ∘-resp-≈ = _ⓘₕ_
}
where open Strong
| {
"alphanum_fraction": 0.5959339263,
"avg_line_length": 33.4893617021,
"ext": "agda",
"hexsha": "4d624704f10bc909a879a4fe3feb502b4354bd89",
"lang": "Agda",
"max_forks_count": 64,
"max_forks_repo_forks_event_max_datetime": "2022-03-14T02:00:59.000Z",
"max_forks_repo_forks_event_min_datetime": "2019-06-02T16:58:15.000Z",
"max_forks_repo_head_hexsha": "d9e4f578b126313058d105c61707d8c8ae987fa8",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "Code-distancing/agda-categories",
"max_forks_repo_path": "src/Categories/Category/Instance/Monoidals.agda",
"max_issues_count": 236,
"max_issues_repo_head_hexsha": "d9e4f578b126313058d105c61707d8c8ae987fa8",
"max_issues_repo_issues_event_max_datetime": "2022-03-28T14:31:43.000Z",
"max_issues_repo_issues_event_min_datetime": "2019-06-01T14:53:54.000Z",
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "Code-distancing/agda-categories",
"max_issues_repo_path": "src/Categories/Category/Instance/Monoidals.agda",
"max_line_length": 72,
"max_stars_count": 279,
"max_stars_repo_head_hexsha": "d9e4f578b126313058d105c61707d8c8ae987fa8",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "Trebor-Huang/agda-categories",
"max_stars_repo_path": "src/Categories/Category/Instance/Monoidals.agda",
"max_stars_repo_stars_event_max_datetime": "2022-03-22T00:40:14.000Z",
"max_stars_repo_stars_event_min_datetime": "2019-06-01T14:36:40.000Z",
"num_tokens": 547,
"size": 1574
} |
module Numeral.FixedPositional where
{-
FixedPositional : ℕ → Type
FixedPositional(b) = List(𝕟(b))
open import Numeral.Natural.Oper
private variable b : ℕ
to-ℕ : FixedPositional(b) → ℕ
to-ℕ {_} ∅ = 𝟎
to-ℕ {b} (n ⊰ l) = 𝕟-to-ℕ (n) + (b ⋅ to-ℕ (l))
-}
{-
module Test2 where
import Lvl
open import Data
open import Data.Boolean hiding (elim)
open import Data.Boolean.Stmt
import Data.Boolean.Operators
open Data.Boolean.Operators.Programming
open import Numeral.Finite
open import Numeral.Natural
open import Functional
open import Syntax.Number
open import Type
open import Type.Dependent
private variable ℓ : Lvl.Level
private variable z : Bool
private variable b n : ℕ
positive? : 𝕟(n) → Bool
positive? 𝟎 = 𝐹
positive? (𝐒 _) = 𝑇
Positive : 𝕟(n) → Type
Positive = IsTrue ∘ positive?
data Positional(b : ℕ) : Type{Lvl.𝟎} where
# : (n : 𝕟(b)) → ⦃ Positive(n) ⦄ → Positional b
_·_ : Positional b → 𝕟(b) → Positional b
infixl 20 _·_
test : Positional 10
test = # 1 · 5 · 0 · 4 · 0 · 0
open import Numeral.Natural.Oper
to-ℕ : Positional b → ℕ
to-ℕ (# n) = 𝕟-to-ℕ n
to-ℕ {b} (l · n) = (b ⋅ (to-ℕ l)) + (to-ℕ (# n))
open import Logic.Propositional
-- open import Numeral.Natural.Decidable
open import Numeral.Natural.Inductions
open import Numeral.Natural.Oper.Comparisons
open import Numeral.Natural.Oper.FlooredDivision
open import Numeral.Natural.Oper.FlooredDivision.Proofs
open import Numeral.Natural.Oper.Modulo
open import Numeral.Natural.Oper.Modulo.Proofs
open import Numeral.Natural.Relation.Order
open import Numeral.Natural.Relation.Order.Decidable
open import Numeral.Natural.Relation.Order.Proofs
open import Structure.Relator.Ordering
open import Type.Properties.Decidable
open import Type.Properties.Decidable.Proofs
from-ℕ-rec : (b : ℕ) → ⦃ b-size : IsTrue(b >? 1) ⦄ → (x : ℕ) → ((prev : ℕ) ⦃ _ : prev < x ⦄ → Positional(b)) → Positional(b)
from-ℕ-rec b@(𝐒(𝐒 _)) 𝟎 _ = intro 𝐹 (# 𝟎)
from-ℕ-rec b@(𝐒(𝐒 _)) n@(𝐒 _) prev with prev(n ⌊/⌋ b) ⦃ [⌊/⌋]-ltₗ {n}{b} ⦄
... | intro 𝑇 r = intro 𝑇 (r · (ℕ-to-𝕟 (n mod b) ⦃ [↔]-to-[→] decider-true (mod-maxᵣ{n}{b}) ⦄))
... | intro 𝐹 r = {!test2 r [≡]-intro!}
from-ℕ : ⦃ b-size : IsTrue(b >? 1) ⦄ → ℕ → Positional(b)
from-ℕ b@{𝐒(𝐒 _)} = Strict.Properties.wellfounded-recursion(_<_) (from-ℕ-rec b)
{-from-ℕ {b = b@(𝐒(𝐒 _))} 𝟎 = intro 𝐹 (# 𝟎)
from-ℕ {b = b@(𝐒(𝐒 _))} n@(𝐒 _) with [<][≥]-dichotomy {n}{b}
... | [∨]-introₗ lt = intro 𝑇 (# (ℕ-to-𝕟 n ⦃ [↔]-to-[→] decider-true lt ⦄))
... | [∨]-introᵣ ge with from-ℕ {b} (n ⌊/⌋ b)
... | intro 𝑇 nb = intro 𝑇 (nb · ℕ-to-𝕟 (n mod b) ⦃ [↔]-to-[→] decider-true (mod-maxᵣ{n}{b}) ⦄)
... | intro 𝐹 _ = intro 𝑇 {!!}-}
-}
module Test where
open import Data.List
open import Numeral.Finite
open import Numeral.Natural
open import Type
open import Numeral.Natural.Oper
private variable b : ℕ
to-ℕ : ℕ → List(ℕ) → ℕ
to-ℕ _ ∅ = 𝟎
to-ℕ b (n ⊰ l) = n + (b ⋅ to-ℕ b l)
module _ where
open import Data
open import Data.Boolean.Stmt
open import Numeral.Natural.Inductions
open import Numeral.Natural.Oper.Comparisons
open import Numeral.Natural.Oper.FlooredDivision
open import Numeral.Natural.Oper.FlooredDivision.Proofs
open import Numeral.Natural.Oper.Modulo
open import Numeral.Natural.Relation
open import Numeral.Natural.Relation.Order
open import Relator.Equals
open import Structure.Relator.Ordering
from-ℕ-rec : (b : ℕ) → ⦃ b-size : IsTrue(b >? 1) ⦄ → (x : ℕ) → ((prev : ℕ) ⦃ _ : prev < x ⦄ → List ℕ) → List ℕ
from-ℕ-rec b@(𝐒(𝐒 _)) 𝟎 _ = ∅
from-ℕ-rec b@(𝐒(𝐒 _)) n@(𝐒 _) prev = (n mod b) ⊰ prev(n ⌊/⌋ b) ⦃ [⌊/⌋]-ltₗ {n} {b} ⦄
from-ℕ : (b : ℕ) → ⦃ b-size : IsTrue(b >? 1) ⦄ → ℕ → List(ℕ)
from-ℕ b@(𝐒(𝐒 _)) = Strict.Properties.wellfounded-recursion(_<_) (from-ℕ-rec b)
open import Numeral.Natural.Oper.DivMod.Proofs
open import Numeral.Natural.Oper.Proofs
open import Structure.Function
open import Structure.Operator
open import Structure.Operator.Properties
open import Syntax.Transitivity
open import Relator.Equals.Proofs.Equiv
to-from-inverse : ∀{b} ⦃ b-size : IsTrue(b >? 1) ⦄ {n} → (to-ℕ b (from-ℕ b n) ≡ n)
to-from-inverse {b@(𝐒(𝐒 bb))} {n} = Strict.Properties.wellfounded-recursion-intro(_<_) {rec = from-ℕ-rec b} {φ = \{n} expr → (to-ℕ b expr ≡ n)} p {n} where
p : (y : ℕ) → _ → _ → (to-ℕ b (Strict.Properties.accessible-recursion(_<_) (from-ℕ-rec b) y) ≡ y)
p 𝟎 _ _ = [≡]-intro
p (𝐒 y) prev step =
to-ℕ b (Strict.Properties.accessible-recursion(_<_) (from-ℕ-rec b) (𝐒 y)) 🝖[ _≡_ ]-[ congruence₁(to-ℕ b) (step {𝐒(y) ⌊/⌋ b} ⦃ [⌊/⌋]-ltₗ {𝐒 y}{b} ⦄) ]
(𝐒(y) mod b) + (b ⋅ to-ℕ b (Strict.Properties.accessible-recursion(_<_) (from-ℕ-rec b) (𝐒(y) ⌊/⌋ b))) 🝖[ _≡_ ]-[ congruence₂ᵣ(_+_)(𝐒(y) mod b) (congruence₂ᵣ(_⋅_)(b) (prev{𝐒(y) ⌊/⌋ b} ⦃ [⌊/⌋]-ltₗ {𝐒 y}{b} ⦄)) ]
(𝐒(y) mod b) + (b ⋅ (𝐒(y) ⌊/⌋ b)) 🝖[ _≡_ ]-[ commutativity(_+_) {𝐒(y) mod b}{b ⋅ (𝐒(y) ⌊/⌋ b)} ]
(b ⋅ (𝐒(y) ⌊/⌋ b)) + (𝐒(y) mod b) 🝖[ _≡_ ]-[ [⌊/⌋][mod]-is-division-with-remainder-pred-commuted {𝐒 y}{b} ]
𝐒(y) 🝖-end
-- TODO: There are some requirements on l for this to hold. For example, it should not end with zeroes (actually start with because the representation is reversed from the usual one), it should not have numbers greater or equal to b
{-from-to-inverse : ∀{b} ⦃ b-size : IsTrue(b >? 1) ⦄ {l} → (from-ℕ b (to-ℕ b l) ≡ l)
from-to-inverse b@{𝐒(𝐒 _)} {l = ∅} = [≡]-intro
from-to-inverse b@{𝐒(𝐒 _)} {l = x ⊰ l} = {!!}-}
{-Strict.Properties.wellfounded-recursion-intro(_<_) {rec = from-ℕ-rec b} {φ = \{n} expr → (expr ≡ from-ℕ b n)} p {x + (b ⋅ to-ℕ b l)} where
p : (y : ℕ) → _ → _ → (Strict.Properties.accessible-recursion(_<_) (from-ℕ-rec b) y ≡ from-ℕ b y)
p 𝟎 prev step = {!!}
p (𝐒 y) prev step = {!!}-}
{-
module _ where
open import Functional
open import Function.Iteration using (repeatᵣ)
open import Numeral.Natural.Induction
open import Relator.Equals
open import Relator.Equals.Proofs
open import Syntax.Function
open import Syntax.Transitivity
{- TODO: Attempt to prove `∀a∀b. aᵇ = 1 + ((a−1) ⋅ ∑(0‥b) (i ↦ aⁱ))` inductively. An intuitive example of this is: `10³ = 1000 = 1+999 = 1+(9⋅111) = 1+(9⋅(1+10+100)) = 1+((10−1)⋅(10⁰+10¹+10²))`. This can also be proved by using the binomial theorem?
powerSum : ℕ → ℕ → ℕ
powerSum a 0 = 0
powerSum a 1 = 1
powerSum a (𝐒(𝐒(b))) = (powerSum a (𝐒(b))) + (a ⋅ (powerSum a (𝐒(b))))
exponentiation-is-sum-of-parts : ∀{a b} → (𝐒(a) ^ b ≡ 𝐒(a ⋅ (powerSum (𝐒(a)) b)))
exponentiation-is-sum-of-parts {a} {0} = [≡]-intro
exponentiation-is-sum-of-parts {a} {1} = [≡]-intro
exponentiation-is-sum-of-parts {a} {𝐒(b@(𝐒(_)))} =
𝐒(a) ^ 𝐒(b) 🝖[ _≡_ ]-[]
𝐒(a) ⋅ (𝐒(a) ^ b) 🝖[ _≡_ ]-[ {!!} ]
(𝐒(a) ^ b) + (𝐒(a) ⋅ (a ⋅ (powerSum (𝐒(a)) b))) 🝖[ _≡_ ]-[ {!!} ]
(𝐒(a) ^ b) + (a ⋅ (𝐒(a) ⋅ (powerSum (𝐒(a)) b))) 🝖[ _≡_ ]-[ {!!} ]
𝐒(a ⋅ (powerSum (𝐒(a)) b)) + (a ⋅ (𝐒(a) ⋅ (powerSum (𝐒(a)) b))) 🝖[ _≡_ ]-[ {!!} ]
𝐒((a ⋅ (powerSum (𝐒(a)) b)) + (a ⋅ (𝐒(a) ⋅ (powerSum (𝐒(a)) b)))) 🝖[ _≡_ ]-[ {!!} ]
𝐒(a ⋅ ((powerSum (𝐒(a)) b) + (𝐒(a) ⋅ (powerSum (𝐒(a)) b)))) 🝖[ _≡_ ]-[]
𝐒(a ⋅ (powerSum (𝐒(a)) (𝐒(b)))) 🝖-end
-}
module _ where
open import Data.List.Functions
open import Numeral.Natural.Relation.Order
open import Numeral.Natural.Relation.Order.Proofs
open import Structure.Relator.Properties
open import Syntax.Transitivity
{-
FixedPositional-maximum : ∀{n : FixedPositional(b)} → (to-ℕ (n) < b ^ length(n))
FixedPositional-maximum {_} {∅} = reflexivity(_≤_)
FixedPositional-maximum {𝐒 b} {n ⊰ l} =
𝐒(𝕟-to-ℕ (n) + (𝐒(b) ⋅ to-ℕ (l))) 🝖[ _≤_ ]-[ {!!} ]
𝐒(𝕟-to-ℕ (n) + (𝐒(b) ⋅ (b ^ length(l)))) 🝖[ _≤_ ]-[ {!!} ]
𝐒(𝕟-to-ℕ (n) + ((b ⋅ (b ^ length(l))) + (1 ⋅ (b ^ length(l))))) 🝖[ _≤_ ]-[ {!!} ]
𝐒(𝕟-to-ℕ (n) + ((b ^ 𝐒(length(l))) + (b ^ length(l)))) 🝖[ _≤_ ]-[ {!!} ]
? 🝖[ _≤_ ]-[ {!!}
(b ⋅ (𝐒(b) ^ length(l))) + (𝐒(b) ^ length(l)) 🝖[ _≤_ ]-[ {!!} ]
𝐒(b) ⋅ (𝐒(b) ^ length(l)) 🝖-end
-}
-}
| {
"alphanum_fraction": 0.5542649302,
"avg_line_length": 43.2639593909,
"ext": "agda",
"hexsha": "b2e2b020981d19040a2ce0d5f3802e2bd389fc34",
"lang": "Agda",
"max_forks_count": null,
"max_forks_repo_forks_event_max_datetime": null,
"max_forks_repo_forks_event_min_datetime": null,
"max_forks_repo_head_hexsha": "70f4fba849f2fd779c5aaa5af122ccb6a5b271ba",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "Lolirofle/stuff-in-agda",
"max_forks_repo_path": "old/Numeral/FixedPositional.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "70f4fba849f2fd779c5aaa5af122ccb6a5b271ba",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "Lolirofle/stuff-in-agda",
"max_issues_repo_path": "old/Numeral/FixedPositional.agda",
"max_line_length": 251,
"max_stars_count": 6,
"max_stars_repo_head_hexsha": "70f4fba849f2fd779c5aaa5af122ccb6a5b271ba",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "Lolirofle/stuff-in-agda",
"max_stars_repo_path": "old/Numeral/FixedPositional.agda",
"max_stars_repo_stars_event_max_datetime": "2022-02-05T06:53:22.000Z",
"max_stars_repo_stars_event_min_datetime": "2020-04-07T17:58:13.000Z",
"num_tokens": 3695,
"size": 8523
} |
module Logic.Predicate.Theorems where
import Lvl
open import Functional
open import Logic
open import Logic.Propositional
open import Logic.Propositional.Theorems
open import Logic.Predicate
open import Syntax.Type
open import Type
open import Type.Properties.Inhabited using (◊ ; [◊]-existence)
------------------------------------------
-- Swapping nested quantifiers
module _ {ℓₒ₁}{ℓₒ₂}{ℓₗ} {X : Type{ℓₒ₁}}{Y : Type{ℓₒ₂}}{P : X → Y → Stmt{ℓₗ}} where
[∀]-swap : ∀ₗ(x ↦ ∀ₗ(y ↦ P(x)(y))) → ∀ₗ(y ↦ ∀ₗ(x ↦ P(x)(y)))
[∀]-swap(xypxy){y}{x} = xypxy{x}{y}
[∃]-swap : ∃(x ↦ ∃(y ↦ P(x)(y))) → ∃(y ↦ ∃(x ↦ P(x)(y)))
[∃]-swap([∃]-intro(x) ⦃ [∃]-intro(y) ⦃ proof ⦄ ⦄) = [∃]-intro(y) ⦃ [∃]-intro(x) ⦃ proof ⦄ ⦄
------------------------------------------
-- Introducing and eliminating unnecessary quantifiers when the predicate is constant
module _ {ℓₒ}{ℓₗ} {X : Type{ℓₒ}} ⦃ pos : ◊ X ⦄ {P : Stmt{ℓₗ}} where
[∃]-unnecessary-intro : P → ∃{Obj = X}(x ↦ P)
[∃]-unnecessary-intro(p) = [∃]-intro([◊]-existence ⦃ pos ⦄) ⦃ p ⦄
module _ {ℓₒ}{ℓₗ} {X : Type{ℓₒ}} {P : Stmt{ℓₗ}} where
[∀]-unnecessary-intro : P → ∀ₗ{Obj = X}(x ↦ P)
[∀]-unnecessary-intro(p){x} = p
[∃]-unnecessary-elim : ∃{Obj = X}(x ↦ P) → P
[∃]-unnecessary-elim([∃]-intro(_) ⦃ proof ⦄) = proof
module _ {ℓₒ}{ℓₗ} {X : Type{ℓₒ}} ⦃ pos : ◊ X ⦄ {P : Stmt{ℓₗ}} where
-- Note:
-- The following is unprovable:
-- [∀]-unnecessary : ∀{X}{P : Stmt} → ∀ₗ{X}(x ↦ P) → P
-- X is not guaranteed to not be the empty type, and even if it was, the ∀ function requires a constructed value. It seems to need a non-empty domain to quantify over.
[∀ₑ]-unnecessary-elim : ∀ₗ{Obj = X}(x ↦ P) → P
[∀ₑ]-unnecessary-elim = [∀ₑ]-elim{Obj = X} ⦃ pos ⦄
------------------------------------------
-- When quantifiers contradict
module _ {ℓₒ}{ℓₗ} {X : Type{ℓₒ}} {P : X → Stmt{ℓₗ}} where
[∀][∃¬]-contradiction : ∀ₗ(x ↦ P(x)) → ∃(x ↦ ¬(P(x))) → ⊥
[∀][∃¬]-contradiction(ap)(enp) =
([∃]-elim(\{a} → np ↦ (
([⊥]-intro
([∀]-elim{Obj = X}{P} ap(a))
np
)
)) (enp))
[∀¬][∃]-contradiction : ∀ₗ(x ↦ ¬ P(x)) → ∃(x ↦ P(x)) → ⊥
[∀¬][∃]-contradiction (axnpx) (expx) =
axnpx {[∃]-witness(expx)} ([∃]-proof(expx))
------------------------------------------
-- Moving in and out negation from quantifiers
module _ {ℓₒ}{ℓₗ} {X : Type{ℓₒ}} {P : X → Stmt{ℓₗ}} where
[∃¬]-to-[¬∀] : (∃(x ↦ ¬(P(x)))) → ¬(∀ₗ(x ↦ P(x)))
[∃¬]-to-[¬∀] = swap ([∀][∃¬]-contradiction {ℓₒ}{ℓₗ})
[∀¬]-to-[¬∃] : ∀ₗ(x ↦ ¬(P(x))) → ¬(∃(x ↦ P(x)))
[∀¬]-to-[¬∃] = [∀¬][∃]-contradiction {ℓₒ}{ℓₗ} {X}{P}
-- [∀¬]-to-[¬∃] (anpx) =
-- ([¬]-intro(epx ↦
-- [∃]-elim(\{a} → pa ↦
-- ([⊥]-intro
-- pa
-- (anpx{a})
-- )
-- )(epx)
-- ))
[¬∃]-to-[∀¬] : ∀ₗ(x ↦ ¬(P(x))) ← ¬(∃(x ↦ P(x)))
[¬∃]-to-[∀¬] (nepx) =
([∀]-intro(a ↦
(([¬]-intro(pa ↦
(([⊥]-intro
(([∃]-intro a ⦃ pa ⦄) :of: (∃(x ↦ P(x))))
(nepx :of: ¬(∃(x ↦ P(x))))
) :of: ⊥)
)) :of: ¬(P(a)))
))
module _ {ℓₒ}{ℓₗ} {X : Type{ℓₒ}} ⦃ pos : ◊ X ⦄ {P : X → Stmt{ℓₗ}} where
[¬∃]-to-[∃¬] : ¬(∃ P) → ∃(¬_ ∘ P)
[¬∃]-to-[∃¬] (nexpx) = [∃]-intro ([◊]-existence ⦃ pos ⦄) ⦃ [¬∃]-to-[∀¬] {ℓₒ}{ℓₗ} {X}{P} (nexpx) ⦄
[¬∃]-to-[¬∀] : ¬(∃ P) → ¬(∀ₗ P)
[¬∃]-to-[¬∀] = ([∃¬]-to-[¬∀] {ℓₒ}{ℓₗ} {X}{P}) ∘ [¬∃]-to-[∃¬]
[∀¬]-to-[¬∀] : ∀ₗ(¬_ ∘ P) → ¬(∀ₗ P)
[∀¬]-to-[¬∀] axnpx axpx = (axnpx{[◊]-existence ⦃ pos ⦄}) (axpx{[◊]-existence ⦃ pos ⦄})
------------------------------------------
-- Introducing negations to change quantifier
module _ {ℓₒ}{ℓₗ} {X : Type{ℓₒ}} {P : X → Stmt{ℓₗ}} where
[∀]-to-[¬∃¬] : ∀ₗ(x ↦ P(x)) → (¬ ∃(x ↦ ¬(P(x))))
[∀]-to-[¬∃¬] = [∀][∃¬]-contradiction {ℓₒ}{ℓₗ} {X}{P} -- [∃]-elim(\{a} → npa ↦ npa(p{a}))(ep)
[∃]-to-[¬∀¬] : ∃(x ↦ P(x)) → (¬ ∀ₗ(x ↦ ¬(P(x))))
[∃]-to-[¬∀¬] = swap ([∀¬][∃]-contradiction {ℓₒ}{ℓₗ} {X}{P})
------------------------------------------
-- Stuff using double negation
module _ {ℓₒ}{ℓₗ} {X : Type{ℓₒ}} {P : X → Stmt{ℓₗ}} where
[∀¬¬][∃¬]-contradiction : ∀ₗ(x ↦ ¬¬(P(x))) → (∃(x ↦ ¬(P(x)))) → ⊥
[∀¬¬][∃¬]-contradiction (annp)([∃]-intro(a) ⦃ na ⦄) =
[∀][∃¬]-contradiction {ℓₒ}{ℓₗ} {X}{¬¬_ ∘ P} (annp)([∃]-intro(a) ⦃ [¬¬]-intro(na) ⦄)
[∀¬¬]-to-[¬∃¬] : ∀ₗ(x ↦ ¬¬(P(x))) → (¬ ∃(x ↦ ¬(P(x))))
[∀¬¬]-to-[¬∃¬] = [∀¬¬][∃¬]-contradiction
[¬¬∀]-to-[¬∃¬] : ¬¬ ∀ₗ(x ↦ (P(x))) → (¬ ∃(x ↦ ¬(P(x))))
[¬¬∀]-to-[¬∃¬] = contrapositiveᵣ ([∃¬]-to-[¬∀] {ℓₒ}{ℓₗ} {X}{P})
-- [¬¬∀]-to-[¬∃¬] (annx) (enx) =
-- ([⊥]-intro
-- ([∃¬]-to-[¬∀](enx))
-- (annx)
-- )
[¬∃¬]-to-[∀¬¬] : ¬(∃(x ↦ ¬(P(x)))) → ∀ₗ(x ↦ ¬¬(P(x)))
[¬∃¬]-to-[∀¬¬] (nenx) {a} (npa) = nenx([∃]-intro(a) ⦃ npa ⦄)
[¬¬∀]-to-[∀¬¬] : ¬¬ ∀ₗ(x ↦ (P(x))) → ∀ₗ(x ↦ ¬¬(P(x)))
[¬¬∀]-to-[∀¬¬] = [¬∃¬]-to-[∀¬¬] ∘ [¬¬∀]-to-[¬∃¬]
[∀]-to-[∃]-conditional-by-existence : ∃(P) → ∀{Q : X → Stmt{ℓₗ}} → ∀ₗ(x ↦ (P(x) → Q(x))) → ∃(x ↦ (P(x) ∧ Q(x)))
∃.witness ([∀]-to-[∃]-conditional-by-existence p pq) = [∃]-witness p
∃.proof ([∀]-to-[∃]-conditional-by-existence p pq) = [∧]-intro ([∃]-proof p) (pq{[∃]-witness p} ([∃]-proof p))
-- TODO: Probably unprovable. Not sure why. Maybe because (¬¬A is valid in constructive logic) ⇔ (A is valid in classical logic), and therefore this would not be possible because everything here is in constructive logic.
-- [∀¬¬]-to-[¬¬∀] : ∀{X}{P : X → Stmt} → ¬¬∀ₗ(x ↦ (P(x))) ← ∀ₗ(x ↦ ¬¬(P(x)))
------------------------------------------
-- Changing quantifier
module _ {ℓₒ}{ℓₗ} {X : Type{ℓₒ}} ⦃ pos : ◊ X ⦄ {P : X → Stmt{ℓₗ}} where
-- Note: If X would be empty, then this would be unprovable because [∀]-elim needs a constructed element.
[∀ₑ]-to-[∃] : ∀ₗ(x ↦ P(x)) → ∃(x ↦ P(x))
[∀ₑ]-to-[∃] (apx) =
[∃]-intro ([◊]-existence ⦃ pos ⦄) ⦃ [∀ₑ]-elim{Obj = X}{P = P}(apx) ⦄
------------------------------------------
-- "Distributing" quantifiers into logical operators
module _ {ℓₒ}{ℓₗ₁}{ℓₗ₂} {X : Type{ℓₒ}}{P : X → Stmt{ℓₗ₁}}{Q : X → Stmt{ℓₗ₂}} where
[∀][→]-distributivity : ∀ₗ(x ↦ (P(x) → Q(x))) → ∀ₗ(x ↦ P(x)) → ∀ₗ(x ↦ Q(x))
[∀][→]-distributivity (PxQx) (Px) = PxQx(Px)
[∀][∧]-distributivity : ∀ₗ(x ↦ (P(x) ∧ Q(x))) ↔ (∀ₗ(x ↦ P(x)) ∧ ∀ₗ(x ↦ Q(x)))
[∀][∧]-distributivity = [↔]-intro l r where
l : (∀ₗ(x ↦ P(x)) ∧ ∀ₗ(x ↦ Q(x))) → ∀ₗ(x ↦ (P(x) ∧ Q(x)))
l ([∧]-intro (axPx) (axQx)) {x} = [∧]-intro (axPx{x}) (axQx{x})
r : (∀ₗ(x ↦ P(x)) ∧ ∀ₗ(x ↦ Q(x))) ← ∀ₗ(x ↦ (P(x) ∧ Q(x)))
r(apxqx) = [∧]-intro (\{x} → [∧]-elimₗ(apxqx{x})) (\{x} → [∧]-elimᵣ(apxqx{x}))
[∃][∨]-distributivity : ∃(x ↦ (P(x) ∨ Q(x))) ↔ (∃(x ↦ P(x)) ∨ ∃(x ↦ Q(x)))
[∃][∨]-distributivity = [↔]-intro l r where
l : (∃(x ↦ P(x)) ∨ ∃(x ↦ Q(x))) → ∃(x ↦ (P(x) ∨ Q(x)))
l ([∨]-introₗ ([∃]-intro x ⦃ px ⦄)) = [∃]-intro x ⦃ [∨]-introₗ px ⦄
l ([∨]-introᵣ ([∃]-intro x ⦃ qx ⦄)) = [∃]-intro x ⦃ [∨]-introᵣ qx ⦄
r : (∃(x ↦ P(x)) ∨ ∃(x ↦ Q(x))) ← ∃(x ↦ (P(x) ∨ Q(x)))
r ([∃]-intro x ⦃ [∨]-introₗ px ⦄) = [∨]-introₗ ([∃]-intro x ⦃ px ⦄)
r ([∃]-intro x ⦃ [∨]-introᵣ qx ⦄) = [∨]-introᵣ ([∃]-intro x ⦃ qx ⦄)
[∃][∧]-semidistributivity : ∃(x ↦ ∃(y ↦ (P(x) ∧ Q(y)))) ↔ (∃(x ↦ P(x)) ∧ ∃(x ↦ Q(x)))
[∃][∧]-semidistributivity = [↔]-intro l r where
l : ∃(x ↦ ∃(y ↦ (P(x) ∧ Q(y)))) ← (∃(x ↦ P(x)) ∧ ∃(x ↦ Q(x)))
l ([∧]-intro ([∃]-intro x ⦃ px ⦄) ([∃]-intro y ⦃ qy ⦄)) = [∃]-intro x ⦃ [∃]-intro y ⦃ [∧]-intro px qy ⦄ ⦄
r : ∃(x ↦ ∃(y ↦ (P(x) ∧ Q(y)))) → (∃(x ↦ P(x)) ∧ ∃(x ↦ Q(x)))
r ([∃]-intro x ⦃ [∃]-intro y ⦃ [∧]-intro px qy ⦄ ⦄) = [∧]-intro ([∃]-intro x ⦃ px ⦄) ([∃]-intro y ⦃ qy ⦄)
[∃][∧]-distributivity : ∃(x ↦ (P(x) ∧ Q(x))) → (∃(x ↦ P(x)) ∧ ∃(x ↦ Q(x)))
[∃][∧]-distributivity ([∃]-intro x ⦃ [∧]-intro px qx ⦄ ) = [∧]-intro l r where
l = [∃]-intro x ⦃ px ⦄
r = [∃]-intro x ⦃ qx ⦄
module _ {ℓₒ}{ℓₗ₁}{ℓₗ₂} {X : Type{ℓₒ}}{P : X → Stmt{ℓₗ₁}}{Q : X → Stmt{ℓₗ₂}} where
[∀][↔]-distributivity : ∀ₗ(x ↦ (P(x) ↔ Q(x))) → (∀ₗ(x ↦ P(x)) ↔ ∀ₗ(x ↦ Q(x)))
[∀][↔]-distributivity = r where -- [↔]-intro l r where
-- l : ∀ₗ(x ↦ (P(x) ↔ Q(x))) ← (∀ₗ(x ↦ P(x)) ↔ ∀ₗ(x ↦ Q(x)))
-- l([↔]-intro aqxapx apxaqx) {x} = [↔]-intro (\qx → aqxpx(qx{x})) (apxqx{x})
r : ∀ₗ(x ↦ (P(x) ↔ Q(x))) → (∀ₗ(x ↦ P(x)) ↔ ∀ₗ(x ↦ Q(x)))
r apxqx = [↔]-intro ([∀][→]-distributivity rl) ([∀][→]-distributivity rr) where
rl : ∀ₗ(x ↦ (P(x) ← Q(x)))
rl{x} = [↔]-to-[←](apxqx{x})
rr : ∀ₗ(x ↦ (P(x) → Q(x)))
rr{x} = [↔]-to-[→](apxqx{x})
[∀]-to-[∃]-[↔]-semidistributivity : ∀ₗ(x ↦ (P(x) ↔ Q(x))) → (∃(x ↦ P(x)) ↔ ∃(x ↦ Q(x)))
[∀]-to-[∃]-[↔]-semidistributivity apq = [↔]-intro ([∃]-map-proof ([↔]-to-[←] apq)) ([∃]-map-proof ([↔]-to-[→] apq))
------------------------------------------
-- Quantifiers with logical operators inside, but one of the predicates are constant
module _ {ℓₒ}{ℓₗ₁}{ℓₗ₂} {X : Type{ℓₒ}}{P : X → Stmt{ℓₗ₁}}{Q : Stmt{ℓₗ₂}} where
[∀]-unrelatedₗ-[→] : ∀ₗ(x ↦ (P(x) → Q)) ↔ (∃(x ↦ P(x)) → Q)
[∀]-unrelatedₗ-[→] = [↔]-intro l r where
l : ∀ₗ(x ↦ (P(x) → Q)) ← (∃(x ↦ P(x)) → Q)
l(expxq) {x} px = expxq([∃]-intro(x) ⦃ px ⦄)
r : ∀ₗ(x ↦ (P(x) → Q)) → (∃(x ↦ P(x)) → Q)
r(axpxq) = [∃]-elim(\{x} → px ↦ axpxq{x}(px))
[∃]-unrelatedₗ-[→]ᵣ : ∃(x ↦ (P(x) → Q)) → (∀ₗ(x ↦ P(x)) → Q)
[∃]-unrelatedₗ-[→]ᵣ = r where -- [↔]-intro l r where
r : ∃(x ↦ (P(x) → Q)) → (∀ₗ(x ↦ P(x)) → Q)
r(expxq)(axpx) = [∃]-proof(expxq) (axpx{[∃]-witness(expxq)})
[∃]-unrelatedₗ-[∧] : ∃(x ↦ (P(x) ∧ Q)) ↔ (∃(x ↦ P(x)) ∧ Q)
[∃]-unrelatedₗ-[∧] = [↔]-intro l r where
l : ∃(x ↦ (P(x) ∧ Q)) ← (∃(x ↦ P(x)) ∧ Q)
l ([∧]-intro ([∃]-intro x ⦃ px ⦄) q) = [∃]-intro x ⦃ [∧]-intro px q ⦄
r : ∃(x ↦ (P(x) ∧ Q)) → (∃(x ↦ P(x)) ∧ Q)
r ([∃]-intro x ⦃ [∧]-intro px q ⦄) = [∧]-intro ([∃]-intro x ⦃ px ⦄) q
module _ {ℓₒ}{ℓₗ₁}{ℓₗ₂} {X : Type{ℓₒ}}{P : Stmt{ℓₗ₁}}{Q : X → Stmt{ℓₗ₂}} where
[∀]-unrelatedᵣ-[→] : ∀ₗ(x ↦ (P → Q(x))) ↔ (P → ∀ₗ(x ↦ Q(x)))
[∀]-unrelatedᵣ-[→] = [↔]-intro l r where
l : ∀ₗ(x ↦ (P → Q(x))) ← (P → ∀ₗ(x ↦ Q(x)))
l(paxqx) {x} p = paxqx(p){x}
r : ∀ₗ(x ↦ (P → Q(x))) → (P → ∀ₗ(x ↦ Q(x)))
r(axpqx)(p){x} = axpqx{x}(p)
[∃]-unrelatedᵣ-[→]ᵣ : ∃(x ↦ (P → Q(x))) → (P → ∃(x ↦ Q(x)))
[∃]-unrelatedᵣ-[→]ᵣ = r where -- [↔]-intro l r where
r : ∃(x ↦ (P → Q(x))) → (P → ∃(x ↦ Q(x)))
r(expqx)(p) = [∃]-elim(\{x} → pqx ↦ [∃]-intro(x) ⦃ pqx(p) ⦄) (expqx)
[∃]-unrelatedᵣ-[∧] : ∃(x ↦ (P ∧ Q(x))) ↔ (P ∧ ∃(x ↦ Q(x)))
[∃]-unrelatedᵣ-[∧] = [↔]-intro l r where
l : ∃(x ↦ (P ∧ Q(x))) ← (P ∧ ∃(x ↦ Q(x)))
l ([∧]-intro p ([∃]-intro x ⦃ qx ⦄)) = [∃]-intro x ⦃ [∧]-intro p qx ⦄
r : ∃(x ↦ (P ∧ Q(x))) → (P ∧ ∃(x ↦ Q(x)))
r ([∃]-intro x ⦃ [∧]-intro p qx ⦄) = [∧]-intro p ([∃]-intro x ⦃ qx ⦄)
------------------------------------------
-- Equivalences
module _ {ℓₒ}{ℓₗ₁}{ℓₗ₂} {X : Type{ℓₒ}}{P : X → Stmt{ℓₗ₁}}{Q : X → Stmt{ℓₗ₂}} where
[∃]-map-proof-[↔] : (∀{x} → P(x) ↔ Q(x)) → ((∃ P) ↔ (∃ Q))
[∃]-map-proof-[↔] p = [↔]-intro ([∃]-map-proof ([↔]-to-[←] p)) ([∃]-map-proof ([↔]-to-[→] p))
------------------------------------------
-- Other rules
module _ {ℓₒ}{ℓₗ₁}{ℓₗ₂} {X : Type{ℓₒ}}{P : X → Stmt{ℓₗ₁}}{Q : X → Stmt{ℓₗ₂}} where
[∀][→]-add-[∃] : ∀ₗ(x ↦ (P(x) → Q(x))) → ∀ₗ(x ↦ (P(x) → ∃(x ↦ Q(x))))
[∀][→]-add-[∃] (proof) {x} px = [∃]-intro(x) ⦃ proof{x} px ⦄
[∀][→]-to-[∃] : ∀ₗ(x ↦ (P(x) → Q(x))) → (∃(x ↦ P(x)) → ∃(x ↦ Q(x)))
[∀][→]-to-[∃] (proof) = ([↔]-to-[→] ([∀]-unrelatedₗ-[→] {X = X} {P})) ([∀][→]-add-[∃] (proof))
module _ {ℓₒ₁}{ℓₒ₂}{ℓₗ} {X : Type{ℓₒ₁}}{Y : Type{ℓₒ₂}}{P : X → Y → Stmt{ℓₗ}} where
[∀][∃]-swap : ∃(x ↦ ∀ₗ(y ↦ P(x)(y))) → ∀ₗ(y ↦ ∃(x ↦ P(x)(y)))
[∀][∃]-swap ([∃]-intro x ⦃ aypxy ⦄) {y} = [∃]-intro x ⦃ aypxy{y} ⦄
{-
no-intermediate : ∀{X : Stmt} → ¬(¬(X ↔ ⊤) ∧ ¬(X ↔ ⊥))
no-intermediate = [¬][∨] [¬¬]-excluded-middle
¬((¬ X) ∧ (¬ Y)) ↔ ¬(¬ (X ∨ Y))
∀{X} → ¬¬(X ∨ (¬ X))
-}
module _ {ℓₒ₁}{ℓₒ₂}{ℓₗ} {X : Type{ℓₒ₁}}{Y : Type{ℓₒ₂}}{P : X → Y → Stmt{ℓₗ}} where
[∀][∃]-to-function-existence : ∀ₗ(x ↦ ∃(y ↦ P(x)(y))) → ∃(f ↦ ∀ₗ(x ↦ P(x)(f(x))))
[∀][∃]-to-function-existence p = [∃]-intro (x ↦ [∃]-witness(p{x})) ⦃ \{x} → [∃]-proof(p{x}) ⦄
| {
"alphanum_fraction": 0.4005492676,
"avg_line_length": 41.8675958188,
"ext": "agda",
"hexsha": "e93422f732410a364bd861cfaa096ab06812c69b",
"lang": "Agda",
"max_forks_count": null,
"max_forks_repo_forks_event_max_datetime": null,
"max_forks_repo_forks_event_min_datetime": null,
"max_forks_repo_head_hexsha": "70f4fba849f2fd779c5aaa5af122ccb6a5b271ba",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "Lolirofle/stuff-in-agda",
"max_forks_repo_path": "Logic/Predicate/Theorems.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "70f4fba849f2fd779c5aaa5af122ccb6a5b271ba",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "Lolirofle/stuff-in-agda",
"max_issues_repo_path": "Logic/Predicate/Theorems.agda",
"max_line_length": 222,
"max_stars_count": 6,
"max_stars_repo_head_hexsha": "70f4fba849f2fd779c5aaa5af122ccb6a5b271ba",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "Lolirofle/stuff-in-agda",
"max_stars_repo_path": "Logic/Predicate/Theorems.agda",
"max_stars_repo_stars_event_max_datetime": "2022-02-05T06:53:22.000Z",
"max_stars_repo_stars_event_min_datetime": "2020-04-07T17:58:13.000Z",
"num_tokens": 6518,
"size": 12016
} |
{-# OPTIONS --sized-types #-}
open import Relation.Binary.Core
module Quicksort.Correctness.Permutation {A : Set}
(_≤_ : A → A → Set)
(tot≤ : Total _≤_) where
open import Bound.Total A
open import Bound.Total.Order _≤_
open import Data.List
open import Data.Product
open import Data.Sum
open import List.Permutation.Base A
open import List.Permutation.Base.Concatenation A
open import List.Permutation.Base.Equivalence A
open import List.Permutation.Pair A
open import List.Permutation.Pair.Properties A
open import Quicksort _≤_ tot≤
open import SBList _≤_
open import SBList.Properties _≤_
open import Size
open import SOList.Total _≤_
lemma-deal : {ι : Size}{b t : Bound}{x : A} → (b≤x : LeB b (val x)) → (x≤t : LeB (val x) t) → (xs : SBList {ι} b t) → unbound xs ≈ unbound× (deal b≤x x≤t xs)
lemma-deal _ _ (nil _) = ≈[]r []
lemma-deal {x = x} b≤x x≤t (cons y b≤y y≤t ys)
with tot≤ x y
... | inj₁ x≤y = ≈xr (lemma-deal b≤x x≤t ys)
... | inj₂ y≤x = ≈xl (lemma-deal b≤x x≤t ys)
lemma-quickSort : {ι : Size}{b t : Bound}(xs : SBList {ι} b t) → unbound xs ∼ forget (quickSort xs)
lemma-quickSort (nil _) = ∼[]
lemma-quickSort (cons x b≤x x≤t xs) = trans∼ (lemma≈∼ (≈xr (lemma-deal b≤x x≤t xs))) (lemma++∼ (lemma-quickSort ys) (∼x /head /head (lemma-quickSort zs)))
where yszs = deal b≤x x≤t xs
ys = proj₁ yszs
zs = proj₂ yszs
theorem-quickSort∼ : (xs : List A) → xs ∼ forget (quickSort (bound xs))
theorem-quickSort∼ xs = trans∼ (lemma-unbound-bound xs) (lemma-quickSort (bound xs))
| {
"alphanum_fraction": 0.6344221106,
"avg_line_length": 38.8292682927,
"ext": "agda",
"hexsha": "0a7022d3189a91bcc395fad9c50eb33b314a7558",
"lang": "Agda",
"max_forks_count": null,
"max_forks_repo_forks_event_max_datetime": null,
"max_forks_repo_forks_event_min_datetime": null,
"max_forks_repo_head_hexsha": "b8d428bccbdd1b13613e8f6ead6c81a8f9298399",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "bgbianchi/sorting",
"max_forks_repo_path": "agda/Quicksort/Correctness/Permutation.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "b8d428bccbdd1b13613e8f6ead6c81a8f9298399",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "bgbianchi/sorting",
"max_issues_repo_path": "agda/Quicksort/Correctness/Permutation.agda",
"max_line_length": 157,
"max_stars_count": 6,
"max_stars_repo_head_hexsha": "b8d428bccbdd1b13613e8f6ead6c81a8f9298399",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "bgbianchi/sorting",
"max_stars_repo_path": "agda/Quicksort/Correctness/Permutation.agda",
"max_stars_repo_stars_event_max_datetime": "2021-08-24T22:11:15.000Z",
"max_stars_repo_stars_event_min_datetime": "2015-05-21T12:50:35.000Z",
"num_tokens": 571,
"size": 1592
} |
{-# OPTIONS --without-K --safe #-}
-- An inhabited Indiscrete category is a -2-Category
module Categories.Minus2-Category.Construction.Indiscrete where
open import Level
open import Data.Unit using (tt)
open import Data.Product using (_,_)
open import Relation.Binary.PropositionalEquality using (refl)
open import Categories.Minus2-Category
open import Categories.Category.Indiscrete
open import Categories.Morphism using (_≅_)
InhIndIs-2 : ∀ {o ℓ} → (X : Set o) → (x : X) → -2-Category {o} {ℓ} {ℓ}
InhIndIs-2 X x = record
{ cat = Indiscrete X
; Obj-Contr = x , λ y → record
{ from = lift tt
; to = lift tt
; iso = record
{ isoˡ = refl
; isoʳ = refl
}
}
; Hom-Conn = refl
}
| {
"alphanum_fraction": 0.6629680999,
"avg_line_length": 25.75,
"ext": "agda",
"hexsha": "4bbb872c92577ccd709cedcf49fdb0fc83f42f95",
"lang": "Agda",
"max_forks_count": 64,
"max_forks_repo_forks_event_max_datetime": "2022-03-14T02:00:59.000Z",
"max_forks_repo_forks_event_min_datetime": "2019-06-02T16:58:15.000Z",
"max_forks_repo_head_hexsha": "d9e4f578b126313058d105c61707d8c8ae987fa8",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "Code-distancing/agda-categories",
"max_forks_repo_path": "src/Categories/Minus2-Category/Construction/Indiscrete.agda",
"max_issues_count": 236,
"max_issues_repo_head_hexsha": "d9e4f578b126313058d105c61707d8c8ae987fa8",
"max_issues_repo_issues_event_max_datetime": "2022-03-28T14:31:43.000Z",
"max_issues_repo_issues_event_min_datetime": "2019-06-01T14:53:54.000Z",
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "Code-distancing/agda-categories",
"max_issues_repo_path": "src/Categories/Minus2-Category/Construction/Indiscrete.agda",
"max_line_length": 70,
"max_stars_count": 279,
"max_stars_repo_head_hexsha": "d9e4f578b126313058d105c61707d8c8ae987fa8",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "Trebor-Huang/agda-categories",
"max_stars_repo_path": "src/Categories/Minus2-Category/Construction/Indiscrete.agda",
"max_stars_repo_stars_event_max_datetime": "2022-03-22T00:40:14.000Z",
"max_stars_repo_stars_event_min_datetime": "2019-06-01T14:36:40.000Z",
"num_tokens": 224,
"size": 721
} |
-- Builtin things aren't allowed inside parameterised modules. It's not clear
-- what that would mean.
module BuiltinInParameterisedModule where
module A (X : Set) where
{-# BUILTIN INTEGER X #-}
| {
"alphanum_fraction": 0.745,
"avg_line_length": 25,
"ext": "agda",
"hexsha": "aeb768a91975b525809e566da3a6e017918f52f6",
"lang": "Agda",
"max_forks_count": 371,
"max_forks_repo_forks_event_max_datetime": "2022-03-30T19:00:30.000Z",
"max_forks_repo_forks_event_min_datetime": "2015-01-03T14:04:08.000Z",
"max_forks_repo_head_hexsha": "231d6ad8e77b67ff8c4b1cb35a6c31ccd988c3e9",
"max_forks_repo_licenses": [
"BSD-3-Clause"
],
"max_forks_repo_name": "Agda-zh/agda",
"max_forks_repo_path": "test/Fail/BuiltinInParameterisedModule.agda",
"max_issues_count": 4066,
"max_issues_repo_head_hexsha": "ed8ac6f4062ea8a20fa0f62d5db82d4e68278338",
"max_issues_repo_issues_event_max_datetime": "2022-03-31T21:14:49.000Z",
"max_issues_repo_issues_event_min_datetime": "2015-01-10T11:24:51.000Z",
"max_issues_repo_licenses": [
"BSD-3-Clause"
],
"max_issues_repo_name": "shlevy/agda",
"max_issues_repo_path": "test/Fail/BuiltinInParameterisedModule.agda",
"max_line_length": 77,
"max_stars_count": 1989,
"max_stars_repo_head_hexsha": "ed8ac6f4062ea8a20fa0f62d5db82d4e68278338",
"max_stars_repo_licenses": [
"BSD-3-Clause"
],
"max_stars_repo_name": "shlevy/agda",
"max_stars_repo_path": "test/Fail/BuiltinInParameterisedModule.agda",
"max_stars_repo_stars_event_max_datetime": "2022-03-30T18:20:48.000Z",
"max_stars_repo_stars_event_min_datetime": "2015-01-09T23:51:16.000Z",
"num_tokens": 48,
"size": 200
} |
{-# OPTIONS --copatterns #-}
module DataRecordCoinductive where
data ⊥ : Set where
record ⊤ : Set where
constructor tt
mutual
data Stream (A : Set) : Set where
cons : Cons A → Stream A
-- since Cons is coinductive, we are creating streams
record Cons (A : Set) : Set where
coinductive
constructor _∷_
field head : A
tail : Stream A
open Cons
mutual
repeat : {A : Set}(a : A) → Stream A
repeat a = cons (repeat' a)
repeat' : {A : Set}(a : A) → Cons A
head (repeat' a) = a
tail (repeat' a) = repeat a
-- should not termination check: coconstructors are not size preserving
consume : {A : Set} → Stream A → ⊥
-- consume (cons s) = consume (tail s) -- fails termination check
consume (cons (x ∷ xs)) = consume xs
loop : ⊥
loop = consume (repeat tt)
| {
"alphanum_fraction": 0.6313823163,
"avg_line_length": 20.075,
"ext": "agda",
"hexsha": "61773dafa9f72d45fdce972f9c4180a1f4bc0429",
"lang": "Agda",
"max_forks_count": 1,
"max_forks_repo_forks_event_max_datetime": "2019-03-05T20:02:38.000Z",
"max_forks_repo_forks_event_min_datetime": "2019-03-05T20:02:38.000Z",
"max_forks_repo_head_hexsha": "6043e77e4a72518711f5f808fb4eb593cbf0bb7c",
"max_forks_repo_licenses": [
"BSD-3-Clause"
],
"max_forks_repo_name": "alhassy/agda",
"max_forks_repo_path": "test/Fail/DataRecordCoinductive.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "6043e77e4a72518711f5f808fb4eb593cbf0bb7c",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"BSD-3-Clause"
],
"max_issues_repo_name": "alhassy/agda",
"max_issues_repo_path": "test/Fail/DataRecordCoinductive.agda",
"max_line_length": 71,
"max_stars_count": 3,
"max_stars_repo_head_hexsha": "6043e77e4a72518711f5f808fb4eb593cbf0bb7c",
"max_stars_repo_licenses": [
"BSD-3-Clause"
],
"max_stars_repo_name": "alhassy/agda",
"max_stars_repo_path": "test/Fail/DataRecordCoinductive.agda",
"max_stars_repo_stars_event_max_datetime": "2015-12-07T20:14:00.000Z",
"max_stars_repo_stars_event_min_datetime": "2015-03-28T14:51:03.000Z",
"num_tokens": 248,
"size": 803
} |
{-# OPTIONS --safe --experimental-lossy-unification #-}
module Cubical.Algebra.Polynomials.UnivariateList.Polyn-nPoly where
open import Cubical.Foundations.Prelude
open import Cubical.Foundations.Equiv
open import Cubical.Data.Nat renaming (_+_ to _+n_; _·_ to _·n_)
open import Cubical.Data.Vec
open import Cubical.Data.Sigma
open import Cubical.Algebra.Ring
open import Cubical.Algebra.CommRing
open import Cubical.Algebra.CommRing.Instances.Polynomials.UnivariatePolyList
open import Cubical.Algebra.CommRing.Instances.Polynomials.MultivariatePoly
open import Cubical.Algebra.Polynomials.Multivariate.EquivCarac.Poly0-A
open import Cubical.Algebra.Polynomials.Multivariate.EquivCarac.An[Am[X]]-Anm[X]
open import Cubical.Algebra.Polynomials.Multivariate.EquivCarac.AB-An[X]Bn[X]
open import Cubical.Algebra.Polynomials.UnivariateList.Poly1-1Poly
open CommRingEquivs renaming (compCommRingEquiv to _∘-ecr_ ; invCommRingEquiv to inv-ecr)
private variable
ℓ : Level
-----------------------------------------------------------------------------
-- Definition
Equiv-Polyn-nPoly : (A' : CommRing ℓ) → (n : ℕ) → CommRingEquiv (PolyCommRing A' n) (nUnivariatePolyList A' n)
Equiv-Polyn-nPoly A' zero = CRE-Poly0-A A'
Equiv-Polyn-nPoly A' (suc n) = inv-ecr _ _ (CRE-PolyN∘M-PolyN+M A' 1 n)
∘-ecr (lift-equiv-poly _ _ 1 (Equiv-Polyn-nPoly A' n)
∘-ecr CRE-Poly1-Poly: (nUnivariatePolyList A' n))
| {
"alphanum_fraction": 0.7098092643,
"avg_line_length": 40.7777777778,
"ext": "agda",
"hexsha": "0e23678764864a5dac08faa2981e0a8ea4ea13ff",
"lang": "Agda",
"max_forks_count": null,
"max_forks_repo_forks_event_max_datetime": null,
"max_forks_repo_forks_event_min_datetime": null,
"max_forks_repo_head_hexsha": "58c0b83bb0fed0dc683f3d29b1709effe51c1689",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "thomas-lamiaux/cubical",
"max_forks_repo_path": "Cubical/Algebra/Polynomials/UnivariateList/Polyn-nPoly.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "58c0b83bb0fed0dc683f3d29b1709effe51c1689",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "thomas-lamiaux/cubical",
"max_issues_repo_path": "Cubical/Algebra/Polynomials/UnivariateList/Polyn-nPoly.agda",
"max_line_length": 110,
"max_stars_count": null,
"max_stars_repo_head_hexsha": "58c0b83bb0fed0dc683f3d29b1709effe51c1689",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "thomas-lamiaux/cubical",
"max_stars_repo_path": "Cubical/Algebra/Polynomials/UnivariateList/Polyn-nPoly.agda",
"max_stars_repo_stars_event_max_datetime": null,
"max_stars_repo_stars_event_min_datetime": null,
"num_tokens": 431,
"size": 1468
} |
------------------------------------------------------------------------------
-- The Booleans
------------------------------------------------------------------------------
{-# OPTIONS --exact-split #-}
{-# OPTIONS --no-sized-types #-}
{-# OPTIONS --no-universe-polymorphism #-}
{-# OPTIONS --without-K #-}
module FOTC.Data.Bool where
open import FOTC.Base
open import FOTC.Data.Bool.Type public
infixr 6 _&&_
------------------------------------------------------------------------------
-- Basic functions
-- The conjunction.
_&&_ : D → D → D
a && b = if a then b else false
{-# ATP definition _&&_ #-}
-- The negation.
not : D → D
not b = if b then false else true
{-# ATP definition not #-}
| {
"alphanum_fraction": 0.3989218329,
"avg_line_length": 25.5862068966,
"ext": "agda",
"hexsha": "e1f4e3d7cfc03f4a1f46691d942d0ad30f107701",
"lang": "Agda",
"max_forks_count": 3,
"max_forks_repo_forks_event_max_datetime": "2018-03-14T08:50:00.000Z",
"max_forks_repo_forks_event_min_datetime": "2016-09-19T14:18:30.000Z",
"max_forks_repo_head_hexsha": "2fc9f2b81052a2e0822669f02036c5750371b72d",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "asr/fotc",
"max_forks_repo_path": "src/fot/FOTC/Data/Bool.agda",
"max_issues_count": 2,
"max_issues_repo_head_hexsha": "2fc9f2b81052a2e0822669f02036c5750371b72d",
"max_issues_repo_issues_event_max_datetime": "2017-01-01T14:34:26.000Z",
"max_issues_repo_issues_event_min_datetime": "2016-10-12T17:28:16.000Z",
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "asr/fotc",
"max_issues_repo_path": "src/fot/FOTC/Data/Bool.agda",
"max_line_length": 78,
"max_stars_count": 11,
"max_stars_repo_head_hexsha": "2fc9f2b81052a2e0822669f02036c5750371b72d",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "asr/fotc",
"max_stars_repo_path": "src/fot/FOTC/Data/Bool.agda",
"max_stars_repo_stars_event_max_datetime": "2021-09-12T16:09:54.000Z",
"max_stars_repo_stars_event_min_datetime": "2015-09-03T20:53:42.000Z",
"num_tokens": 139,
"size": 742
} |
module Let where
f
: {A : Set}
→ A
→ A
f x
= let
y = x
z = x
in y
| {
"alphanum_fraction": 0.3586956522,
"avg_line_length": 7.0769230769,
"ext": "agda",
"hexsha": "96b6a1d5cda05486bdcdef8be9e238ae31149afe",
"lang": "Agda",
"max_forks_count": 1,
"max_forks_repo_forks_event_max_datetime": "2022-03-01T16:38:14.000Z",
"max_forks_repo_forks_event_min_datetime": "2022-03-01T16:38:14.000Z",
"max_forks_repo_head_hexsha": "f327f9aab8dcb07022b857736d8201906bba02e9",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "msuperdock/agda-unused",
"max_forks_repo_path": "data/expression/Let.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "f327f9aab8dcb07022b857736d8201906bba02e9",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "msuperdock/agda-unused",
"max_issues_repo_path": "data/expression/Let.agda",
"max_line_length": 16,
"max_stars_count": 6,
"max_stars_repo_head_hexsha": "f327f9aab8dcb07022b857736d8201906bba02e9",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "msuperdock/agda-unused",
"max_stars_repo_path": "data/expression/Let.agda",
"max_stars_repo_stars_event_max_datetime": "2022-03-01T16:38:05.000Z",
"max_stars_repo_stars_event_min_datetime": "2020-10-29T09:38:43.000Z",
"num_tokens": 42,
"size": 92
} |
module Sections where
open import Haskell.Prelude
test₁ : Nat → Nat
test₁ = 5 +_
test₂ : Nat → Nat
test₂ = _+ 5
test₃ : Nat → Nat
test₃ = _+_ 5
test₄ : Nat → Nat
test₄ = λ x → x + 5
test₅ : Nat → Nat
test₅ = λ x → 5 + x -- Agda eta-contracts this before we get to see it
{-# COMPILE AGDA2HS test₁ #-}
{-# COMPILE AGDA2HS test₂ #-}
{-# COMPILE AGDA2HS test₃ #-}
{-# COMPILE AGDA2HS test₄ #-}
{-# COMPILE AGDA2HS test₅ #-}
| {
"alphanum_fraction": 0.6317016317,
"avg_line_length": 16.5,
"ext": "agda",
"hexsha": "7c4e8877154ebb92385ed5de241f88bd103400bf",
"lang": "Agda",
"max_forks_count": 18,
"max_forks_repo_forks_event_max_datetime": "2022-03-12T11:42:52.000Z",
"max_forks_repo_forks_event_min_datetime": "2020-10-21T22:19:09.000Z",
"max_forks_repo_head_hexsha": "160478a51bc78b0fdab07b968464420439f9fed6",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "seanpm2001/agda2hs",
"max_forks_repo_path": "test/Sections.agda",
"max_issues_count": 63,
"max_issues_repo_head_hexsha": "160478a51bc78b0fdab07b968464420439f9fed6",
"max_issues_repo_issues_event_max_datetime": "2022-02-25T15:47:30.000Z",
"max_issues_repo_issues_event_min_datetime": "2020-10-22T05:19:27.000Z",
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "seanpm2001/agda2hs",
"max_issues_repo_path": "test/Sections.agda",
"max_line_length": 70,
"max_stars_count": 55,
"max_stars_repo_head_hexsha": "8c8f24a079ed9677dbe6893cf786e7ed52dfe8b6",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "dxts/agda2hs",
"max_stars_repo_path": "test/Sections.agda",
"max_stars_repo_stars_event_max_datetime": "2022-03-26T21:57:56.000Z",
"max_stars_repo_stars_event_min_datetime": "2020-10-20T13:36:25.000Z",
"num_tokens": 163,
"size": 429
} |
{-# OPTIONS --without-K --exact-split --safe #-}
open import Fragment.Equational.Theory
module Fragment.Equational.Coproduct (Θ : Theory) where
open import Fragment.Equational.Model Θ
open import Fragment.Algebra.Homomorphism (Σ Θ)
open import Level using (Level; Setω)
private
variable
a b c ℓ₁ ℓ₂ ℓ₃ : Level
module _
(A : Model {a} {ℓ₁})
(B : Model {b} {ℓ₂})
(A+B : Model {c} {ℓ₃})
where
record IsCoproduct : Setω where
field
inl : ∥ A ∥ₐ ⟿ ∥ A+B ∥ₐ
inr : ∥ B ∥ₐ ⟿ ∥ A+B ∥ₐ
_[_,_] : ∀ {d ℓ₄} (X : Model {d} {ℓ₄})
→ ∥ A ∥ₐ ⟿ ∥ X ∥ₐ
→ ∥ B ∥ₐ ⟿ ∥ X ∥ₐ
→ ∥ A+B ∥ₐ ⟿ ∥ X ∥ₐ
commute₁ : ∀ {d ℓ₄} {X : Model {d} {ℓ₄}}
→ {f : ∥ A ∥ₐ ⟿ ∥ X ∥ₐ}
→ {g : ∥ B ∥ₐ ⟿ ∥ X ∥ₐ}
→ X [ f , g ] ⊙ inl ≗ f
commute₂ : ∀ {d ℓ₄} {X : Model {d} {ℓ₄}}
→ {f : ∥ A ∥ₐ ⟿ ∥ X ∥ₐ}
→ {g : ∥ B ∥ₐ ⟿ ∥ X ∥ₐ}
→ X [ f , g ] ⊙ inr ≗ g
universal : ∀ {d ℓ₄} {X : Model {d} {ℓ₄}}
→ {f : ∥ A ∥ₐ ⟿ ∥ X ∥ₐ}
→ {g : ∥ B ∥ₐ ⟿ ∥ X ∥ₐ}
→ {h : ∥ A+B ∥ₐ ⟿ ∥ X ∥ₐ}
→ h ⊙ inl ≗ f
→ h ⊙ inr ≗ g
→ X [ f , g ] ≗ h
| {
"alphanum_fraction": 0.3739266198,
"avg_line_length": 26.1428571429,
"ext": "agda",
"hexsha": "11004e4eb090bfc3b13a6977c9bdc7336cb956c3",
"lang": "Agda",
"max_forks_count": 3,
"max_forks_repo_forks_event_max_datetime": "2021-06-16T08:04:31.000Z",
"max_forks_repo_forks_event_min_datetime": "2021-06-15T15:34:50.000Z",
"max_forks_repo_head_hexsha": "f2a6b1cf4bc95214bd075a155012f84c593b9496",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "yallop/agda-fragment",
"max_forks_repo_path": "src/Fragment/Equational/Coproduct.agda",
"max_issues_count": 1,
"max_issues_repo_head_hexsha": "f2a6b1cf4bc95214bd075a155012f84c593b9496",
"max_issues_repo_issues_event_max_datetime": "2021-06-16T10:24:15.000Z",
"max_issues_repo_issues_event_min_datetime": "2021-06-16T09:44:31.000Z",
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "yallop/agda-fragment",
"max_issues_repo_path": "src/Fragment/Equational/Coproduct.agda",
"max_line_length": 55,
"max_stars_count": 18,
"max_stars_repo_head_hexsha": "f2a6b1cf4bc95214bd075a155012f84c593b9496",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "yallop/agda-fragment",
"max_stars_repo_path": "src/Fragment/Equational/Coproduct.agda",
"max_stars_repo_stars_event_max_datetime": "2022-01-17T17:26:09.000Z",
"max_stars_repo_stars_event_min_datetime": "2021-06-15T15:45:39.000Z",
"num_tokens": 577,
"size": 1281
} |
-- Parametrised maps of families and their coalgebraic properties
module SOAS.Coalgebraic.Map {T : Set} where
open import SOAS.Common
open import SOAS.Context
open import SOAS.Variable
open import SOAS.Families.Core {T}
open import SOAS.Abstract.Hom {T}
import SOAS.Abstract.Box {T} as □ ; open □.Sorted
import SOAS.Abstract.Coalgebra {T} as →□ ; open →□.Sorted
private
variable
𝒳 𝒴 𝒫 : Familyₛ
Γ Δ Θ : Ctx
α : T
record Coalgebraic (𝒳ᴮ : Coalgₚ 𝒳)(𝒫ᴮ : Coalgₚ 𝒫)(𝒴ᴮ : Coalgₚ 𝒴)
(f : 𝒳 ⇾̣ 〖 𝒫 , 𝒴 〗) : Set where
private module 𝒳 = Coalgₚ 𝒳ᴮ
private module 𝒫 = Coalgₚ 𝒫ᴮ
private module 𝒴 = Coalgₚ 𝒴ᴮ
-- Interaction between the point and renaming of all three coalgebras
field
r∘f : {σ : Γ ~[ 𝒫 ]↝ Δ}{ϱ : Δ ↝ Θ}{t : 𝒳 α Γ}
→ 𝒴.r (f t σ) ϱ ≡ f t (λ v → 𝒫.r (σ v) ϱ)
f∘r : {ρ : Γ ↝ Δ}{ς : Δ ~[ 𝒫 ]↝ Θ}{t : 𝒳 α Γ}
→ f (𝒳.r t ρ) ς ≡ f t (ς ∘ ρ)
f∘η : {v : ℐ α Γ} → f (𝒳.η v) 𝒫.η ≡ 𝒴.η v
-- Codomain of coalgebraic map is a pointed coalgebra
〖𝒫,𝒴〗ᴮ : Coalgₚ 〖 𝒫 , 𝒴 〗
〖𝒫,𝒴〗ᴮ = record
{ ᵇ = record { r = λ h ρ σ → h (σ ∘ ρ) ; counit = refl ; comult = refl }
; η = λ v σ → f (𝒳.η v) σ
; r∘η = dext (λ σ → trans (sym f∘r) (congr 𝒳.r∘η (λ - → f - σ))) }
-- The map is a pointed coalgebra homomorphism
ᴮ⇒ : Coalgₚ⇒ 𝒳ᴮ 〖𝒫,𝒴〗ᴮ f
ᴮ⇒ = record { ᵇ⇒ = record { ⟨r⟩ = dext′ f∘r } ; ⟨η⟩ = refl }
-- Equality of two substitutions at the new index extends to equality of
-- transforming new variables with the substitution
eq-at-new : {σ : α ∙ Γ ~[ 𝒫 ]↝ α ∙ Θ}
{ς : α ∙ Δ ~[ 𝒫 ]↝ α ∙ Θ}
→ σ new ≡ ς new
→ f (𝒳.η new) σ ≡ f (𝒳.η new) ς
eq-at-new {σ = σ} {ς} eq = begin
f (𝒳.η new) σ ≡⟨⟩
f (𝒳.η (ι new)) σ ≡˘⟨ cong (λ - → f - σ) (𝒳.r∘η) ⟩
f (𝒳.r (𝒳.η new) ι) σ ≡⟨ f∘r ⟩
f (𝒳.η new) (σ ∘ ι) ≡⟨ cong (f (𝒳.η new)) (dext (λ{ new → eq })) ⟩
f (𝒳.η new) (ς ∘ ι) ≡˘⟨ f∘r ⟩
f (𝒳.r (𝒳.η new) ι) ς ≡⟨ cong (λ - → f - ς) (𝒳.r∘η) ⟩
f (𝒳.η (ι new)) ς ≡⟨⟩
f (𝒳.η new) ς ∎
where
open ≡-Reasoning
open Coalgₚ
ι : (α ∙ ∅) ↝ (α ∙ Δ)
ι new = new
-- Application for a pointed coalgebra is coalgebraic
jᶜ : (𝒳ᴮ : Coalgₚ 𝒳) → Coalgebraic ℐᴮ 𝒳ᴮ 𝒳ᴮ (j 𝒳)
jᶜ 𝒳ᴮ = record { r∘f = refl ; f∘r = refl ; f∘η = refl }
-- Renaming of pointed coalgebr is coalgebraic
rᶜ : (𝒳ᴮ : Coalgₚ 𝒳) → Coalgebraic 𝒳ᴮ ℐᴮ 𝒳ᴮ (Coalgₚ.r 𝒳ᴮ)
rᶜ 𝒳ᴮ = record { r∘f = sym comult ; f∘r = sym comult ; f∘η = r∘η }
where open Coalgₚ 𝒳ᴮ
| {
"alphanum_fraction": 0.5163450177,
"avg_line_length": 33.8533333333,
"ext": "agda",
"hexsha": "40c3fa104a8966850bc2168214f046198974e218",
"lang": "Agda",
"max_forks_count": 4,
"max_forks_repo_forks_event_max_datetime": "2022-01-24T12:49:17.000Z",
"max_forks_repo_forks_event_min_datetime": "2021-11-09T20:39:59.000Z",
"max_forks_repo_head_hexsha": "ff1a985a6be9b780d3ba2beff68e902394f0a9d8",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "JoeyEremondi/agda-soas",
"max_forks_repo_path": "SOAS/Coalgebraic/Map.agda",
"max_issues_count": 1,
"max_issues_repo_head_hexsha": "ff1a985a6be9b780d3ba2beff68e902394f0a9d8",
"max_issues_repo_issues_event_max_datetime": "2021-11-21T12:19:32.000Z",
"max_issues_repo_issues_event_min_datetime": "2021-11-21T12:19:32.000Z",
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "JoeyEremondi/agda-soas",
"max_issues_repo_path": "SOAS/Coalgebraic/Map.agda",
"max_line_length": 78,
"max_stars_count": 39,
"max_stars_repo_head_hexsha": "ff1a985a6be9b780d3ba2beff68e902394f0a9d8",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "JoeyEremondi/agda-soas",
"max_stars_repo_path": "SOAS/Coalgebraic/Map.agda",
"max_stars_repo_stars_event_max_datetime": "2022-03-19T17:33:12.000Z",
"max_stars_repo_stars_event_min_datetime": "2021-11-09T20:39:55.000Z",
"num_tokens": 1351,
"size": 2539
} |
------------------------------------------------------------------------
-- The Agda standard library
--
-- Strings: builtin type and basic operations
------------------------------------------------------------------------
{-# OPTIONS --without-K --safe #-}
module Data.String.Base where
open import Level using (zero)
open import Data.Bool using (true; false)
open import Data.Nat.Base as ℕ using (ℕ; _∸_; ⌊_/2⌋; ⌈_/2⌉)
import Data.Nat.Properties as ℕₚ
open import Data.List.Base as List using (List; [_])
open import Data.List.NonEmpty as NE using (List⁺)
open import Data.List.Extrema ℕₚ.≤-totalOrder
open import Data.List.Relation.Binary.Pointwise using (Pointwise)
open import Data.List.Relation.Binary.Lex.Strict using (Lex-<)
open import Data.Vec.Base as Vec using (Vec)
open import Data.Char.Base as Char using (Char)
import Data.Char.Properties as Char using (_≟_)
open import Function
open import Relation.Binary using (Rel)
open import Relation.Nullary using (does)
open import Data.List.Membership.DecPropositional Char._≟_
------------------------------------------------------------------------
-- From Agda.Builtin: type and renamed primitives
-- Note that we do not re-export primStringAppend because we want to
-- give it an infix definition and be able to assign it a level.
import Agda.Builtin.String as String
open String public using ( String )
renaming
( primStringToList to toList
; primStringFromList to fromList
; primShowString to show
)
------------------------------------------------------------------------
-- Relations
-- Pointwise equality on Strings
infix 4 _≈_
_≈_ : Rel String zero
_≈_ = Pointwise Char._≈_ on toList
-- Lexicographic ordering on Strings
infix 4 _<_
_<_ : Rel String zero
_<_ = Lex-< Char._≈_ Char._<_ on toList
------------------------------------------------------------------------
-- Operations
-- Additional conversion functions
fromChar : Char → String
fromChar = fromList ∘′ [_]
fromList⁺ : List⁺ Char → String
fromList⁺ = fromList ∘′ NE.toList
-- List-like functions
infixr 5 _++_
_++_ : String → String → String
_++_ = String.primStringAppend
length : String → ℕ
length = List.length ∘ toList
replicate : ℕ → Char → String
replicate n = fromList ∘ List.replicate n
concat : List String → String
concat = List.foldr _++_ ""
intersperse : String → List String → String
intersperse sep = concat ∘′ (List.intersperse sep)
-- String-specific functions
unlines : List String → String
unlines = intersperse "\n"
unwords : List String → String
unwords = intersperse " "
parens : String → String
parens s = "(" ++ s ++ ")"
-- enclose string with parens if it contains a space character
parensIfSpace : String → String
parensIfSpace s with does (' ' ∈? toList s)
... | true = parens s
... | false = s
braces : String → String
braces s = "{" ++ s ++ "}"
-- append that also introduces spaces, if necessary
infixr 5 _<+>_
_<+>_ : String → String → String
"" <+> b = b
a <+> "" = a
a <+> b = a ++ " " ++ b
------------------------------------------------------------------------
-- Padding
-- Each one of the padding functions should verify the following
-- invariant:
-- If length str ≤ n then length (padLeft c n str) ≡ n
-- and otherwise padLeft c n str ≡ str.
-- Appending an empty string is expensive (append for Haskell's
-- Text creates a fresh Text value in which both contents are
-- copied) so we precompute `n ∸ length str` and check whether
-- it is equal to 0.
padLeft : Char → ℕ → String → String
padLeft c n str with n ∸ length str
... | 0 = str
... | l = replicate l c ++ str
padRight : Char → ℕ → String → String
padRight c n str with n ∸ length str
... | 0 = str
... | l = str ++ replicate l c
padBoth : Char → Char → ℕ → String → String
padBoth cₗ cᵣ n str with n ∸ length str
... | 0 = str
... | l = replicate ⌊ l /2⌋ cₗ ++ str ++ replicate ⌈ l /2⌉ cᵣ
------------------------------------------------------------------------
-- Alignment
-- We can align a String left, center or right in a column of a given
-- width by padding it with whitespace.
data Alignment : Set where
Left Center Right : Alignment
fromAlignment : Alignment → ℕ → String → String
fromAlignment Left = padRight ' '
fromAlignment Center = padBoth ' ' ' '
fromAlignment Right = padLeft ' '
------------------------------------------------------------------------
-- Rectangle
-- Build a rectangular column by:
-- Given a vector of cells and a padding function for each one
-- Compute the max of the widths, and pad the strings accordingly.
rectangle : ∀ {n} → Vec (ℕ → String → String) n →
Vec String n → Vec String n
rectangle pads cells = Vec.zipWith (λ p c → p width c) pads cells where
sizes = List.map length (Vec.toList cells)
width = max 0 sizes
-- Special cases for left, center, and right alignment
rectangleˡ : ∀ {n} → Char → Vec String n → Vec String n
rectangleˡ c = rectangle (Vec.replicate $ padLeft c)
rectangleʳ : ∀ {n} → Char → Vec String n → Vec String n
rectangleʳ c = rectangle (Vec.replicate $ padRight c)
rectangleᶜ : ∀ {n} → Char → Char → Vec String n → Vec String n
rectangleᶜ cₗ cᵣ = rectangle (Vec.replicate $ padBoth cₗ cᵣ)
| {
"alphanum_fraction": 0.6145974126,
"avg_line_length": 28.6132596685,
"ext": "agda",
"hexsha": "3ca454b9b333c0716b3b60c25ed4071f83b3fa11",
"lang": "Agda",
"max_forks_count": 1,
"max_forks_repo_forks_event_max_datetime": "2021-11-04T06:54:45.000Z",
"max_forks_repo_forks_event_min_datetime": "2021-11-04T06:54:45.000Z",
"max_forks_repo_head_hexsha": "fb380f2e67dcb4a94f353dbaec91624fcb5b8933",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "DreamLinuxer/popl21-artifact",
"max_forks_repo_path": "agda-stdlib/src/Data/String/Base.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "fb380f2e67dcb4a94f353dbaec91624fcb5b8933",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "DreamLinuxer/popl21-artifact",
"max_issues_repo_path": "agda-stdlib/src/Data/String/Base.agda",
"max_line_length": 72,
"max_stars_count": 5,
"max_stars_repo_head_hexsha": "fb380f2e67dcb4a94f353dbaec91624fcb5b8933",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "DreamLinuxer/popl21-artifact",
"max_stars_repo_path": "agda-stdlib/src/Data/String/Base.agda",
"max_stars_repo_stars_event_max_datetime": "2020-10-10T21:41:32.000Z",
"max_stars_repo_stars_event_min_datetime": "2020-10-07T12:07:53.000Z",
"num_tokens": 1342,
"size": 5179
} |
{-# OPTIONS --cubical --safe --postfix-projections #-}
module Data.Array where
open import Data.Binary
open import Prelude
private
variable
ns : 𝔹
record 2× {a} (A : Type a) : Type a where
eta-equality
constructor _⊛_
field
pr₁ pr₂ : A
open 2× public
infixr 5 _∷₁_ _∷₂_ _∷_
mutual
record Array0ᵇ {a} : Type a where
eta-equality
constructor []
record Array1ᵇ {a} (A : Type a) (ns : 𝔹) : Type a where
eta-equality
inductive
constructor _∷₁_
field
head1ᵇ : A
tail1ᵇ : Array (2× A) ns
record Array2ᵇ {a} (A : Type a) (ns : 𝔹) : Type a where
eta-equality
inductive
constructor _∷₂_
field
head2ᵇ : 2× A
tail2ᵇ : Array (2× A) ns
Array : Type a → 𝔹 → Type a
Array A 0ᵇ = Array0ᵇ
Array A (1ᵇ ns) = Array1ᵇ A ns
Array A (2ᵇ ns) = Array2ᵇ A ns
_∷_ : A → Array A ns → Array A (inc ns)
_∷_ {ns = 0ᵇ} x xs = x ∷₁ xs
_∷_ {ns = 1ᵇ ns} x₁ (x₂ ∷₁ xs) = (x₁ ⊛ x₂) ∷₂ xs
_∷_ {ns = 2ᵇ ns} x₁ (x₂ ∷₂ xs) = x₁ ∷₁ x₂ ∷ xs
open import Lens
⦅head1ᵇ⦆ : Lens (Array A (1ᵇ ns)) A
⦅head1ᵇ⦆ .fst (x ∷₁ xs) = lens-part x (_∷₁ xs)
⦅head1ᵇ⦆ .snd .get-set xs v i = v
⦅head1ᵇ⦆ .snd .set-get xs i = xs
⦅head1ᵇ⦆ .snd .set-set (x ∷₁ xs) v₁ v₂ i = v₂ ∷₁ xs
⦅head2ᵇ⦆ : Lens (Array A (2ᵇ ns)) (2× A)
⦅head2ᵇ⦆ .fst (x ∷₂ xs) = lens-part x (_∷₂ xs)
⦅head2ᵇ⦆ .snd .get-set (x ∷₂ xs) v i = v
⦅head2ᵇ⦆ .snd .set-get (x ∷₂ xs) i = x ∷₂ xs
⦅head2ᵇ⦆ .snd .set-set (x ∷₂ xs) v₁ v₂ i = v₂ ∷₂ xs
⦅tail1ᵇ⦆ : Lens (Array A (1ᵇ ns)) (Array (2× A) ns)
⦅tail1ᵇ⦆ .fst (x ∷₁ xs) = lens-part xs (x ∷₁_)
⦅tail1ᵇ⦆ .snd .get-set (x ∷₁ xs) v i = v
⦅tail1ᵇ⦆ .snd .set-get (x ∷₁ xs) i = x ∷₁ xs
⦅tail1ᵇ⦆ .snd .set-set (x ∷₁ xs) v₁ v₂ i = x ∷₁ v₂
⦅tail2ᵇ⦆ : Lens (Array A (2ᵇ ns)) (Array (2× A) ns)
⦅tail2ᵇ⦆ .fst (x ∷₂ xs) = lens-part xs (x ∷₂_)
⦅tail2ᵇ⦆ .snd .get-set (x ∷₂ xs) v i = v
⦅tail2ᵇ⦆ .snd .set-get (x ∷₂ xs) i = x ∷₂ xs
⦅tail2ᵇ⦆ .snd .set-set (x ∷₂ xs) v₁ v₂ i = x ∷₂ v₂
⦅pr₁⦆ : Lens (2× A) A
⦅pr₁⦆ .fst (x ⊛ y) = lens-part x (_⊛ y)
⦅pr₁⦆ .snd .get-set s v i = v
⦅pr₁⦆ .snd .set-get s i = s
⦅pr₁⦆ .snd .set-set s v₁ v₂ i = v₂ ⊛ s .pr₂
⦅pr₂⦆ : Lens (2× A) A
⦅pr₂⦆ .fst (x ⊛ y) = lens-part y (x ⊛_)
⦅pr₂⦆ .snd .get-set s v i = v
⦅pr₂⦆ .snd .set-get s i = s
⦅pr₂⦆ .snd .set-set s v₁ v₂ i = s .pr₁ ⊛ v₂
open import Data.Binary.Order
mutual
index : ∀ is {js} → is < js → Lens (Array A js) A
index 0ᵇ {1ᵇ js} p = ⦅head1ᵇ⦆
index 0ᵇ {2ᵇ js} p = ⦅head2ᵇ⦆ ⋯ ⦅pr₁⦆
index (1ᵇ is) {js} p = ind₂1ᵇ is p
index (2ᵇ is) {1ᵇ js} p = ⦅tail1ᵇ⦆ ⋯ index is p ⋯ ⦅pr₂⦆
index (2ᵇ is) {2ᵇ js} p = ⦅tail2ᵇ⦆ ⋯ index is p ⋯ ⦅pr₁⦆
ind₂1ᵇ : ∀ is {js} → 1ᵇ is < js → Lens (Array A js) A
ind₂1ᵇ is {1ᵇ js} p = ⦅tail1ᵇ⦆ ⋯ index is p ⋯ ⦅pr₁⦆
ind₂1ᵇ 0ᵇ {2ᵇ js} p = ⦅head2ᵇ⦆ ⋯ ⦅pr₂⦆
ind₂1ᵇ (1ᵇ is) {2ᵇ js} p = ⦅tail2ᵇ⦆ ⋯ ind₃ is p ⋯ ⦅pr₂⦆
ind₂1ᵇ (2ᵇ is) {2ᵇ js} p = ⦅tail2ᵇ⦆ ⋯ ind₂2ᵇ is p ⋯ ⦅pr₂⦆
ind₂2ᵇ : ∀ is {js} → 2ᵇ is ≤ js → Lens (Array A js) A
ind₂2ᵇ is {1ᵇ js} p = ⦅tail1ᵇ⦆ ⋯ index is p ⋯ ⦅pr₁⦆
ind₂2ᵇ 0ᵇ {2ᵇ js} p = ⦅head2ᵇ⦆ ⋯ ⦅pr₂⦆
ind₂2ᵇ (1ᵇ is) {2ᵇ js} p = ⦅tail2ᵇ⦆ ⋯ ind₃ is p ⋯ ⦅pr₂⦆
ind₂2ᵇ (2ᵇ is) {2ᵇ js} p = ⦅tail2ᵇ⦆ ⋯ ind₂2ᵇ is p ⋯ ⦅pr₂⦆
ind₃ : ∀ is {js} → 1ᵇ is ≤ js → Lens (Array A js) A
ind₃ 0ᵇ {1ᵇ js} p = ⦅head1ᵇ⦆
ind₃ 0ᵇ {2ᵇ js} p = ⦅head2ᵇ⦆ ⋯ ⦅pr₁⦆
ind₃ (1ᵇ is) {1ᵇ js} p = ⦅tail1ᵇ⦆ ⋯ ind₃ is p ⋯ ⦅pr₂⦆
ind₃ (1ᵇ is) {2ᵇ js} p = ⦅tail2ᵇ⦆ ⋯ ind₃ is p ⋯ ⦅pr₁⦆
ind₃ (2ᵇ is) {1ᵇ js} p = ⦅tail1ᵇ⦆ ⋯ ind₂2ᵇ is p ⋯ ⦅pr₂⦆
ind₃ (2ᵇ is) {2ᵇ js} p = ⦅tail2ᵇ⦆ ⋯ ind₂2ᵇ is p ⋯ ⦅pr₁⦆
at : ∀ is {js} → {p : is < js} → Lens (Array A js) A
at is {p = p} = index is p
import Data.Nat as ℕ
foldrP : ∀ {p} (P : ℕ → Type p) → (∀ {n} → A → P n → P (suc n)) → P zero → Array A ns → P ⟦ ns ⇓⟧
foldrP {ns = 0ᵇ} P f b [] = b
foldrP {ns = 1ᵇ ns} P f b (x ∷₁ xs) = f x (foldrP (λ n → P (n ℕ.* 2)) (λ { (x₁ ⊛ x₂) b → f x₁ (f x₂ b) }) b xs)
foldrP {ns = 2ᵇ ns} P f b ((x₁ ⊛ x₂) ∷₂ xs) = f x₁ (f x₂ (foldrP (λ n → P (n ℕ.* 2)) (λ { (x₁ ⊛ x₂) b → f x₁ (f x₂ b)}) b xs))
foldr : (A → B → B) → B → Array A ns → B
foldr f b = foldrP (λ _ → _) f b
map : (A → B) → Array A ns → Array B ns
map {ns = 0ᵇ} f xs = []
map {ns = 1ᵇ ns} f (x ∷₁ xs) = f x ∷₁ map (λ { (x₁ ⊛ x₂) → f x₁ ⊛ f x₂ }) xs
map {ns = 2ᵇ ns} f ((x₁ ⊛ x₂) ∷₂ xs) = (f x₁ ⊛ f x₂) ∷₂ map (λ { (x₁ ⊛ x₂) → f x₁ ⊛ f x₂ }) xs
import Data.List as List
open import Data.List using (List)
toList : Array A ns → List.List A
toList = foldr List._∷_ List.[]
fromList : (xs : List A) → Array A ⟦ List.length xs ⇑⟧
fromList List.[] = []
fromList (x List.∷ xs) = x ∷ fromList xs
-- Lens laws are satisfied definitionally:
-- get-set
_ : (xs : Array ℕ ⟦ 10 ⇑⟧) (n : ℕ) → (xs [ at ⟦ 5 ⇑⟧ ]≔ n [ at ⟦ 5 ⇑⟧ ]) ≡ n
_ = λ xs n → refl
-- set-get
_ : (xs : Array ℕ ⟦ 10 ⇑⟧) → (xs [ at ⟦ 5 ⇑⟧ ]≔ (xs [ at ⟦ 5 ⇑⟧ ])) ≡ xs
_ = λ xs → refl
-- set-set
_ : (xs : Array ℕ ⟦ 10 ⇑⟧) (n m : ℕ) → (xs [ at ⟦ 5 ⇑⟧ ]≔ n [ at ⟦ 5 ⇑⟧ ]≔ m) ≡ (xs [ at ⟦ 5 ⇑⟧ ]≔ m)
_ = λ xs n m → refl
| {
"alphanum_fraction": 0.5255785627,
"avg_line_length": 30.5962732919,
"ext": "agda",
"hexsha": "68eefa73ebcda4ab879f53a40e0ef809a35a986e",
"lang": "Agda",
"max_forks_count": 1,
"max_forks_repo_forks_event_max_datetime": "2021-11-11T12:30:21.000Z",
"max_forks_repo_forks_event_min_datetime": "2021-11-11T12:30:21.000Z",
"max_forks_repo_head_hexsha": "97a3aab1282b2337c5f43e2cfa3fa969a94c11b7",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "oisdk/agda-playground",
"max_forks_repo_path": "Data/Array.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "97a3aab1282b2337c5f43e2cfa3fa969a94c11b7",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "oisdk/agda-playground",
"max_issues_repo_path": "Data/Array.agda",
"max_line_length": 126,
"max_stars_count": 6,
"max_stars_repo_head_hexsha": "97a3aab1282b2337c5f43e2cfa3fa969a94c11b7",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "oisdk/agda-playground",
"max_stars_repo_path": "Data/Array.agda",
"max_stars_repo_stars_event_max_datetime": "2021-11-16T08:11:34.000Z",
"max_stars_repo_stars_event_min_datetime": "2020-09-11T17:45:41.000Z",
"num_tokens": 3016,
"size": 4926
} |
{- Byzantine Fault Tolerant Consensus Verification in Agda, version 0.9.
Copyright (c) 2021, Oracle and/or its affiliates.
Licensed under the Universal Permissive License v 1.0 as shown at https://opensource.oracle.com/licenses/upl
-}
import LibraBFT.Impl.Consensus.ConsensusTypes.VoteData as VoteData
open import LibraBFT.Impl.OBM.Crypto hiding (verify)
open import LibraBFT.Impl.OBM.Logging.Logging
import LibraBFT.Impl.Types.ValidatorVerifier as ValidatorVerifier
open import LibraBFT.ImplShared.Consensus.Types
open import Optics.All
open import Util.Hash
open import Util.PKCS hiding (verify)
open import Util.Prelude
------------------------------------------------------------------------------
open import Data.String using (String)
module LibraBFT.Impl.Consensus.ConsensusTypes.Vote where
------------------------------------------------------------------------------
timeout : Vote → Timeout
------------------------------------------------------------------------------
newWithSignature : VoteData → Author → LedgerInfo → Signature → Vote
newWithSignature voteData author ledgerInfo signature =
Vote∙new voteData author ledgerInfo signature nothing
verify : Vote → ValidatorVerifier → Either ErrLog Unit
verify self validator = do
lcheck (self ^∙ vLedgerInfo ∙ liConsensusDataHash == hashVD (self ^∙ vVoteData))
(here' ("Vote's hash mismatch with LedgerInfo" ∷ []))
withErrCtx' (here' ("vote" ∷ []))
(ValidatorVerifier.verify validator (self ^∙ vAuthor) (self ^∙ vLedgerInfo) (self ^∙ vSignature))
case self ^∙ vTimeoutSignature of λ where
nothing → pure unit
(just tos) →
withErrCtx' (here' ("timeout" ∷ []))
(ValidatorVerifier.verify validator (self ^∙ vAuthor) (timeout self) tos)
withErrCtx' (here' ("VoteData" ∷ [])) (VoteData.verify (self ^∙ vVoteData))
where
here' : List String → List String
here' t = "Vote" ∷ "verify" ∷ "failed" {-∷lsV self-} ∷ t
addTimeoutSignature : Vote → Signature → Vote
addTimeoutSignature self sig =
if is-just (self ^∙ vTimeoutSignature)
then self
else self & vTimeoutSignature ?~ sig
timeout v =
Timeout∙new (v ^∙ vVoteData ∙ vdProposed ∙ biEpoch) (v ^∙ vVoteData ∙ vdProposed ∙ biRound)
isTimeout : Vote → Bool
isTimeout v = is-just (v ^∙ vTimeoutSignature)
| {
"alphanum_fraction": 0.6243760399,
"avg_line_length": 39.4098360656,
"ext": "agda",
"hexsha": "9027f675a70fe198689e81f8917150ffbbe4b1f7",
"lang": "Agda",
"max_forks_count": null,
"max_forks_repo_forks_event_max_datetime": null,
"max_forks_repo_forks_event_min_datetime": null,
"max_forks_repo_head_hexsha": "a4674fc473f2457fd3fe5123af48253cfb2404ef",
"max_forks_repo_licenses": [
"UPL-1.0"
],
"max_forks_repo_name": "LaudateCorpus1/bft-consensus-agda",
"max_forks_repo_path": "src/LibraBFT/Impl/Consensus/ConsensusTypes/Vote.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "a4674fc473f2457fd3fe5123af48253cfb2404ef",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"UPL-1.0"
],
"max_issues_repo_name": "LaudateCorpus1/bft-consensus-agda",
"max_issues_repo_path": "src/LibraBFT/Impl/Consensus/ConsensusTypes/Vote.agda",
"max_line_length": 111,
"max_stars_count": null,
"max_stars_repo_head_hexsha": "a4674fc473f2457fd3fe5123af48253cfb2404ef",
"max_stars_repo_licenses": [
"UPL-1.0"
],
"max_stars_repo_name": "LaudateCorpus1/bft-consensus-agda",
"max_stars_repo_path": "src/LibraBFT/Impl/Consensus/ConsensusTypes/Vote.agda",
"max_stars_repo_stars_event_max_datetime": null,
"max_stars_repo_stars_event_min_datetime": null,
"num_tokens": 606,
"size": 2404
} |
------------------------------------------------------------------------
-- The Agda standard library
--
-- Instantiates the ring solver, using the natural numbers as the
-- coefficient "ring"
------------------------------------------------------------------------
open import Algebra
import Algebra.Operations
open import Relation.Nullary
module Algebra.RingSolver.Natural-coefficients
{r₁ r₂}
(R : CommutativeSemiring r₁ r₂)
(dec : let open CommutativeSemiring R
open Algebra.Operations semiring in
∀ m n → Dec (m × 1# ≈ n × 1#)) where
import Algebra.RingSolver
open import Algebra.RingSolver.AlmostCommutativeRing
open import Data.Nat as ℕ
open import Data.Product using (module Σ)
open import Function
import Relation.Binary.EqReasoning
import Relation.Nullary.Decidable as Dec
open CommutativeSemiring R
open Algebra.Operations semiring
open Relation.Binary.EqReasoning setoid
private
-- The coefficient "ring".
ℕ-ring : RawRing _
ℕ-ring = record
{ Carrier = ℕ
; _+_ = ℕ._+_
; _*_ = ℕ._*_
; -_ = id
; 0# = 0
; 1# = 1
}
-- There is a homomorphism from ℕ to R.
--
-- Note that _×′_ is used rather than _×_. If _×_ were used, then
-- Function.Related.TypeIsomorphisms.test would fail to type-check.
homomorphism :
ℕ-ring -Raw-AlmostCommutative⟶ fromCommutativeSemiring R
homomorphism = record
{ ⟦_⟧ = λ n → n ×′ 1#
; +-homo = ×′-homo-+ 1#
; *-homo = ×′1-homo-*
; -‿homo = λ _ → refl
; 0-homo = refl
; 1-homo = refl
}
-- Equality of certain expressions can be decided.
dec′ : ∀ m n → Dec (m ×′ 1# ≈ n ×′ 1#)
dec′ m n = Dec.map′ to from (dec m n)
where
to : m × 1# ≈ n × 1# → m ×′ 1# ≈ n ×′ 1#
to m≈n = begin
m ×′ 1# ≈⟨ sym $ ×≈×′ m 1# ⟩
m × 1# ≈⟨ m≈n ⟩
n × 1# ≈⟨ ×≈×′ n 1# ⟩
n ×′ 1# ∎
from : m ×′ 1# ≈ n ×′ 1# → m × 1# ≈ n × 1#
from m≈n = begin
m × 1# ≈⟨ ×≈×′ m 1# ⟩
m ×′ 1# ≈⟨ m≈n ⟩
n ×′ 1# ≈⟨ sym $ ×≈×′ n 1# ⟩
n × 1# ∎
-- The instantiation.
open Algebra.RingSolver _ _ homomorphism dec′ public
| {
"alphanum_fraction": 0.52677747,
"avg_line_length": 26.0963855422,
"ext": "agda",
"hexsha": "971b68a4cd2e88a8435ae9dc038ecaf1aacbff0e",
"lang": "Agda",
"max_forks_count": null,
"max_forks_repo_forks_event_max_datetime": null,
"max_forks_repo_forks_event_min_datetime": null,
"max_forks_repo_head_hexsha": "9d4c43b1609d3f085636376fdca73093481ab882",
"max_forks_repo_licenses": [
"Apache-2.0"
],
"max_forks_repo_name": "qwe2/try-agda",
"max_forks_repo_path": "agda-stdlib-0.9/src/Algebra/RingSolver/Natural-coefficients.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "9d4c43b1609d3f085636376fdca73093481ab882",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"Apache-2.0"
],
"max_issues_repo_name": "qwe2/try-agda",
"max_issues_repo_path": "agda-stdlib-0.9/src/Algebra/RingSolver/Natural-coefficients.agda",
"max_line_length": 72,
"max_stars_count": 1,
"max_stars_repo_head_hexsha": "9d4c43b1609d3f085636376fdca73093481ab882",
"max_stars_repo_licenses": [
"Apache-2.0"
],
"max_stars_repo_name": "qwe2/try-agda",
"max_stars_repo_path": "agda-stdlib-0.9/src/Algebra/RingSolver/Natural-coefficients.agda",
"max_stars_repo_stars_event_max_datetime": "2016-10-20T15:52:05.000Z",
"max_stars_repo_stars_event_min_datetime": "2016-10-20T15:52:05.000Z",
"num_tokens": 762,
"size": 2166
} |
------------------------------------------------------------------------
-- Definitions of combinatorial functions
------------------------------------------------------------------------
{-# OPTIONS --without-K --safe --exact-split #-}
module Math.Combinatorics.Function where
-- agda-stdlib
import Algebra.Operations.CommutativeMonoid as CommutativeMonoidOperations
open import Data.Fin using (toℕ)
open import Data.Nat
open import Data.Nat.DivMod
open import Data.Nat.Properties using (+-0-commutativeMonoid)
open import Data.List
open import Data.Sum using (_⊎_; inj₁; inj₂)
open import Data.Unit using (tt)
open import Relation.Binary.PropositionalEquality
open import Relation.Nullary using (yes; no; ¬_)
open import Relation.Nullary.Decidable using (False; fromWitnessFalse)
-- agda-misc
open import Math.NumberTheory.Summation.Nat
open CommutativeMonoidOperations +-0-commutativeMonoid
infix 10 _! _!!
------------------------------------------------------------------------
-- Factorial
-- n ! = n * (n - 1) * ... * 2 * 1
-- A000142
_! : ℕ → ℕ
0 ! = 1
(suc n) ! = suc n * n !
------------------------------------------------------------------------
-- Permutation, Falling factorial
-- P n k = (n)ₖ = n * (n - 1) * ... * (n - k + 1) (k terms)
P : ℕ → ℕ → ℕ
P n 0 = 1
P 0 (suc k) = 0
P (suc n) (suc k) = suc n * P n k
------------------------------------------------------------------------
-- Combination, Binomial coefficient
-- C n k = P n k / k !
C : ℕ → ℕ → ℕ
C n 0 = 1
C 0 (suc k) = 0
C (suc n) (suc k) = (C n k * suc n) / suc k
-- recursive definition
CRec : ℕ → ℕ → ℕ
CRec n 0 = 1
CRec 0 (suc k) = 0
CRec (suc n) (suc k) = CRec n k + CRec n (suc k)
------------------------------------------------------------------------
-- Double factorial
-- A006882
_!! : ℕ → ℕ
0 !! = 1
1 !! = 1
suc (suc n) !! = suc (suc n) * n !!
------------------------------------------------------------------------
-- unsigned Stirling numbers of the first kind
S1 : ℕ → ℕ → ℕ
S1 0 0 = 1
S1 0 (suc k) = 0
S1 (suc n) 0 = 0
S1 (suc n) (suc k) = n * S1 n (suc k) + S1 n k
------------------------------------------------------------------------
-- Stirling numbers of the second kind
S2 : ℕ → ℕ → ℕ
S2 0 0 = 1
S2 0 (suc k) = 0
S2 (suc n) 0 = 0
S2 (suc n) (suc k) = suc k * S2 n (suc k) + S2 n k
------------------------------------------------------------------------
-- Lah number
L : ℕ → ℕ → ℕ
L n 0 = 0
L 0 (suc k) = 0
L 1 1 = 1
L 1 (suc (suc k)) = 0
L (suc n@(suc _)) (suc k) = (n + suc k) * L n (suc k) + L n k
------------------------------------------------------------------------
-- Bell number
-- A000110
B : ℕ → ℕ
B n = Σ[ i ≤ n ] S2 n i
------------------------------------------------------------------------
-- Pochhammer symbol, Rising factorial
-- Poch n k = x^(n) = n * (n + 1) * ... * (n + k - 1) (k terms)
Poch : ℕ → ℕ → ℕ
Poch n 0 = 1
Poch n (suc k) = n * Poch (suc n) k
------------------------------------------------------------------------
-- Central binomial coefficient
-- A000984
CB : ℕ → ℕ
CB n = C (2 * n) n
------------------------------------------------------------------------
-- Catalan number
-- A000108
Catalan : ℕ → ℕ
Catalan n = CB n / suc n
------------------------------------------------------------------------
-- Eulerian number
A : ℕ → ℕ → ℕ
A 0 0 = 1
A 0 (suc m) = 0
A (suc n) 0 = 1
A (suc n) (suc m) = (n ∸ m) * A n m + suc (suc m) * A n (suc m)
------------------------------------------------------------------------
-- Eulerian numbers of the second kind
E2 : ℕ → ℕ → ℕ
E2 0 0 = 1
E2 0 (suc m) = 0
E2 (suc n) 0 = 1
E2 (suc n) (suc m) =
(2 * suc n ∸ suc m ∸ 1) * E2 n m + suc (suc m) * E2 n (suc m)
------------------------------------------------------------------------
-- Multinomial coefficient
-- Multinomial xs = (sum xs) ! / product (map _! xs)
Multinomial : List ℕ → ℕ
Multinomial [] = 1
Multinomial xxs@(x ∷ xs) = C (sum xxs) x * Multinomial xs
------------------------------------------------------------------------
-- Pascal's triangle
gpascal : ∀ {a} {A : Set a} → (A → A → A) → A → A → ℕ → List A
gpascal f v0 v1 0 = v1 ∷ []
gpascal f v0 v1 (suc n) =
let ps = gpascal f v0 v1 n in zipWith f (v0 ∷ ps) (ps ∷ʳ v0)
pascal : ℕ → List ℕ
pascal = gpascal _+_ 0 1
| {
"alphanum_fraction": 0.3866138265,
"avg_line_length": 27.5272727273,
"ext": "agda",
"hexsha": "f124f23fd575d227a21201b24ea5d6fcc01df3bc",
"lang": "Agda",
"max_forks_count": null,
"max_forks_repo_forks_event_max_datetime": null,
"max_forks_repo_forks_event_min_datetime": null,
"max_forks_repo_head_hexsha": "9fafa35c940ff7b893a80120f6a1f22b0a3917b7",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "rei1024/agda-combinatorics",
"max_forks_repo_path": "Math/Combinatorics/Function.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "9fafa35c940ff7b893a80120f6a1f22b0a3917b7",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "rei1024/agda-combinatorics",
"max_issues_repo_path": "Math/Combinatorics/Function.agda",
"max_line_length": 74,
"max_stars_count": 3,
"max_stars_repo_head_hexsha": "9fafa35c940ff7b893a80120f6a1f22b0a3917b7",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "rei1024/agda-combinatorics",
"max_stars_repo_path": "Math/Combinatorics/Function.agda",
"max_stars_repo_stars_event_max_datetime": "2020-04-25T07:25:27.000Z",
"max_stars_repo_stars_event_min_datetime": "2019-06-25T08:24:15.000Z",
"num_tokens": 1387,
"size": 4542
} |
{-# OPTIONS --without-K --safe #-}
module Source.Size.Substitution.Canonical where
open import Source.Size
open import Util.Prelude
infix 0 Sub⊢
infixl 5 _>>_
data Sub (Δ : Ctx) : (Ω : Ctx) → Set where
[] : Sub Δ []
Snoc : (σ : Sub Δ Ω) (n : Size Δ) → Sub Δ (Ω ∙ m)
variable
σ τ σ′ τ′ ι ι′ : Sub Δ Ω
subV : Sub Δ Ω → Var Ω → Size Δ
subV (Snoc σ n) zero = n
subV (Snoc σ n) (suc x) = subV σ x
sub : Sub Δ Ω → Size Ω → Size Δ
sub σ (var x) = subV σ x
sub σ ∞ = ∞
sub σ zero = zero
sub σ (suc n) = suc (sub σ n)
data Sub⊢ Δ : ∀ Ω (σ : Sub Δ Ω) → Set where
[] : Sub⊢ Δ [] []
Snoc : (⊢σ : Sub⊢ Δ Ω σ) (n<m : n < sub σ m) → Sub⊢ Δ (Ω ∙ m) (Snoc σ n)
syntax Sub⊢ Δ Ω σ = σ ∶ Δ ⇒ Ω
abstract
sub-Snoc : ∀ (σ : Sub Δ Ω) n o
→ sub (Snoc {m = m} σ n) (wk o) ≡ sub σ o
sub-Snoc σ n (var x) = refl
sub-Snoc σ n ∞ = refl
sub-Snoc σ n zero = refl
sub-Snoc σ n (suc o) = cong suc (sub-Snoc σ n o)
mutual
subV-resp-< : σ ∶ Δ ⇒ Ω → var x < n → subV σ x < sub σ n
subV-resp-< {x = zero} (Snoc {σ = σ} {n} {m} ⊢σ n<m) (var refl)
= subst (n <_) (sym (sub-Snoc σ n m)) n<m
subV-resp-< {x = suc x} (Snoc {σ = σ} {n} {m} ⊢σ n<m) (var refl)
= subst (subV σ x <_) (sym (sub-Snoc σ n (bound x)))
(subV-resp-< ⊢σ (var refl))
subV-resp-< ⊢σ <suc = <suc
subV-resp-< ⊢σ (<-trans x<m m<n)
= <-trans (subV-resp-< ⊢σ x<m) (sub-resp-< ⊢σ m<n)
sub-resp-< : σ ∶ Δ ⇒ Ω → n < m → sub σ n < sub σ m
sub-resp-< ⊢σ (var p) = subV-resp-< ⊢σ (var p)
sub-resp-< ⊢σ zero<suc = zero<suc
sub-resp-< ⊢σ zero<∞ = zero<∞
sub-resp-< ⊢σ (suc<suc n<m) = suc<suc (sub-resp-< ⊢σ n<m)
sub-resp-< ⊢σ (suc<∞ n<∞) = suc<∞ (sub-resp-< ⊢σ n<∞)
sub-resp-< ⊢σ (<-trans n<o o<m)
= <-trans (sub-resp-< ⊢σ n<o) (sub-resp-< ⊢σ o<m)
sub-resp-< ⊢σ <suc = <suc
Weaken : Sub Δ Ω → Sub (Δ ∙ n) Ω
Weaken [] = []
Weaken (Snoc σ m) = Snoc (Weaken σ) (wk m)
abstract
subV-Weaken : ∀ (σ : Sub Δ Ω) x → subV (Weaken {n = o} σ) x ≡ wk (subV σ x)
subV-Weaken (Snoc σ n) zero = refl
subV-Weaken (Snoc σ n) (suc x) = subV-Weaken σ x
sub-Weaken : ∀ (σ : Sub Δ Ω) n → sub (Weaken {n = o} σ) n ≡ wk (sub σ n)
sub-Weaken σ (var x) = subV-Weaken σ x
sub-Weaken σ ∞ = refl
sub-Weaken σ zero = refl
sub-Weaken σ (suc n) = cong suc (sub-Weaken σ n)
Weaken⊢ : σ ∶ Δ ⇒ Ω → Weaken σ ∶ Δ ∙ n ⇒ Ω
Weaken⊢ [] = []
Weaken⊢ (Snoc {σ = σ} {n} {m} ⊢σ n<m)
= Snoc (Weaken⊢ ⊢σ)
(subst (wk n <_) (sym (sub-Weaken σ m)) (wk-resp-< n<m))
Lift : (σ : Sub Δ Ω) → Sub (Δ ∙ m) (Ω ∙ n)
Lift σ = Snoc (Weaken σ) (var zero)
abstract
Lift⊢ : σ ∶ Δ ⇒ Ω → m ≡ sub σ n → Lift σ ∶ Δ ∙ m ⇒ Ω ∙ n
Lift⊢ {Δ} {σ = σ} {n = n} ⊢σ refl
= Snoc (Weaken⊢ ⊢σ) (var (sub-Weaken σ n))
mutual
Id : Sub Δ Δ
Id {[]} = []
Id {Δ ∙ n} = Lift Id
abstract
subV-Id : ∀ x → subV (Id {Δ}) x ≡ var x
subV-Id zero = refl
subV-Id (suc x) = trans (subV-Weaken Id x) (cong wk (subV-Id x))
sub-Id : ∀ n → σ ≡ Id → sub σ n ≡ n
sub-Id (var x) refl = subV-Id x
sub-Id ∞ _ = refl
sub-Id zero _ = refl
sub-Id (suc n) p = cong suc (sub-Id n p)
abstract
Id⊢ : Id ∶ Δ ⇒ Δ
Id⊢ {[]} = []
Id⊢ {Δ ∙ n} = Lift⊢ Id⊢ (sym (sub-Id _ refl))
Wk : Sub (Δ ∙ n) Δ
Wk = Weaken Id
abstract
sub-Wk : ∀ n → sub (Wk {Δ} {o}) n ≡ wk n
sub-Wk n = trans (sub-Weaken Id n) (cong wk (sub-Id _ refl))
Wk⊢ : Wk ∶ Δ ∙ n ⇒ Δ
Wk⊢ = Weaken⊢ Id⊢
Sing : Size Δ → Sub Δ (Δ ∙ m)
Sing n = Snoc Id n
abstract
Sing⊢ : n < m → Sing n ∶ Δ ⇒ Δ ∙ m
Sing⊢ {n = n} n<m
= Snoc Id⊢ (subst (n <_) (sym (sub-Id _ refl)) n<m)
_>>_ : Sub Δ Δ′ → Sub Δ′ Δ″ → Sub Δ Δ″
σ >> [] = []
σ >> Snoc τ n = Snoc (σ >> τ) (sub σ n)
abstract
subV->> : ∀ (σ : Sub Δ Δ′) (τ : Sub Δ′ Δ″) x
→ subV (σ >> τ) x ≡ sub σ (subV τ x)
subV->> σ (Snoc τ n) zero = refl
subV->> σ (Snoc τ n) (suc x) = subV->> σ τ x
sub->> : ∀ n → ι ≡ σ >> τ
→ sub ι n ≡ sub σ (sub τ n)
sub->> {σ = σ} {τ} (var x) refl = subV->> σ τ x
sub->> ∞ _ = refl
sub->> zero _ = refl
sub->> (suc n) p = cong suc (sub->> n p)
sub->>′ : σ >> τ ≡ σ′ >> τ′ → sub σ (sub τ n) ≡ sub σ′ (sub τ′ n)
sub->>′ {σ = σ} {τ = τ} {σ′ = σ′} {τ′} {n} eq
= trans (sym (sub->> n refl))
(trans (cong (λ σ → sub σ n) eq) (sub->> n refl))
>>⊢ : σ ∶ Δ ⇒ Δ′ → τ ∶ Δ′ ⇒ Δ″ → σ >> τ ∶ Δ ⇒ Δ″
>>⊢ ⊢σ [] = []
>>⊢ {σ = σ} ⊢σ (Snoc {σ = τ} {n} {m} ⊢τ n<m)
= Snoc (>>⊢ ⊢σ ⊢τ)
(subst (sub σ n <_) (sym (sub->> m refl)) (sub-resp-< ⊢σ n<m))
Skip : Sub (Δ ∙ n ∙ v0) (Δ ∙ n)
Skip = Snoc (Weaken Wk) (var zero)
abstract
Skip⊢ : Skip ∶ Δ ∙ n ∙ v0 ⇒ Δ ∙ n
Skip⊢ {n = n}
= Snoc (Weaken⊢ Wk⊢)
(<-trans (var refl)
(var (trans (sub-Weaken Wk n) (cong wk (sub-Wk n)))))
Weaken>> : Weaken σ >> τ ≡ Weaken {n = n} (σ >> τ)
Weaken>> {τ = []} = refl
Weaken>> {σ = σ} {τ = Snoc τ n} = cong₂ Snoc Weaken>> (sub-Weaken σ n)
Snoc>>Weaken : Snoc {m = m} σ n >> Weaken τ ≡ σ >> τ
Snoc>>Weaken {τ = []} = refl
Snoc>>Weaken {σ = σ} {n = n} {τ = Snoc τ k}
= cong₂ Snoc Snoc>>Weaken (sub-Snoc σ n k)
id-l : Id >> σ ≡ σ
id-l {σ = []} = refl
id-l {σ = Snoc σ n} = cong₂ Snoc id-l (sub-Id n refl)
id-r : {σ : Sub Δ Ω} → σ >> Id ≡ σ
id-r {σ = []} = refl
id-r {σ = Snoc σ n} = cong₂ Snoc (trans Snoc>>Weaken id-r) refl
>>-assoc : σ >> (τ >> ι) ≡ σ >> τ >> ι
>>-assoc {ι = []} = refl
>>-assoc {σ = σ} {τ = τ} {ι = Snoc ι n}
= cong₂ Snoc >>-assoc (sym (sub->> n refl))
Wk>> : Wk >> σ ≡ Weaken {n = n} σ
Wk>> = trans Weaken>> (cong Weaken id-l)
Snoc>>Wk : Snoc {m = m} σ n >> Wk ≡ σ
Snoc>>Wk = trans Snoc>>Weaken id-r
Lift>>Weaken : Lift {m = m} {n} σ >> Weaken τ ≡ Weaken (σ >> τ)
Lift>>Weaken = trans Snoc>>Weaken Weaken>>
Lift>>Wk : Lift {m = m} {n} σ >> Wk ≡ Wk >> σ
Lift>>Wk = trans Lift>>Weaken (trans (sym Wk>>) (cong (Wk >>_) id-r))
Sing>>Weaken : Sing {m = m} n >> Weaken σ ≡ σ
Sing>>Weaken = trans Snoc>>Weaken id-l
Sing>>Wk : Sing {m = m} n >> Wk ≡ Id
Sing>>Wk = trans Snoc>>Weaken id-r
Sing>>Lift : ∀ n → Sing (sub σ n) >> Lift {m = m} {o} σ ≡ σ >> Sing n
Sing>>Lift n = cong₂ Snoc (trans Sing>>Weaken (sym id-r)) refl
Lift>>Lift : Lift {m = m} {n} σ >> Lift {n = o} τ ≡ Lift (σ >> τ)
Lift>>Lift = cong₂ Snoc Lift>>Weaken refl
Skip>>Weaken : Skip {n = n} >> Weaken σ ≡ Weaken (Weaken σ)
Skip>>Weaken = trans Snoc>>Weaken (trans Weaken>> (cong Weaken Wk>>))
Skip>>Lift : Skip >> Lift {m = m} {n} σ ≡ Lift (Lift σ) >> Skip
Skip>>Lift
= cong₂ Snoc
(trans Skip>>Weaken
(sym (trans Lift>>Weaken (cong Weaken (trans Snoc>>Weaken id-r)))))
refl
Lift-Id : Lift {m = m} Id ≡ Id
Lift-Id = refl
LiftSing>>Wk>>Wk : Lift {m = o} {m} (Sing n) >> (Wk >> Wk) ≡ Wk
LiftSing>>Wk>>Wk {n = n} = let open ≡-Reasoning in
begin
Lift (Sing n) >> (Wk >> Wk)
≡⟨ cong (Lift (Sing n) >>_) Wk>> ⟩
Lift (Sing n) >> (Weaken Wk)
≡⟨ Lift>>Weaken ⟩
Weaken (Sing n >> Weaken Id)
≡⟨ cong Weaken Sing>>Weaken ⟩
Wk
∎
LiftSing>>Skip
: Lift {m = m} (Sing {m = m} n) >> Skip ≡ Sing {m = o} (var zero) >> Lift Wk
LiftSing>>Skip {n = n} = cong₂ Snoc go refl
where
go : Lift (Sing n) >> Weaken Wk ≡ Sing (var zero) >> Weaken Wk
go = let open ≡-Reasoning in
begin
Lift (Sing n) >> Weaken Wk
≡⟨ Lift>>Weaken ⟩
Weaken (Sing n >> Weaken Id)
≡⟨ cong Weaken Sing>>Wk ⟩
Wk
≡⟨ sym Sing>>Weaken ⟩
Sing (var zero) >> Weaken Wk
∎
LiftLift>>Skip : Lift (Lift {m = m} {n} σ) >> Skip ≡ Skip >> Lift σ
LiftLift>>Skip
= cong₂ Snoc (trans Lift>>Weaken
(sym (trans Skip>>Weaken (cong Weaken (sym Snoc>>Wk))))) refl
| {
"alphanum_fraction": 0.4895132056,
"avg_line_length": 24.9161290323,
"ext": "agda",
"hexsha": "d2cc48852d485bd177910aa072a127d0e02529bc",
"lang": "Agda",
"max_forks_count": null,
"max_forks_repo_forks_event_max_datetime": null,
"max_forks_repo_forks_event_min_datetime": null,
"max_forks_repo_head_hexsha": "104cddc6b65386c7e121c13db417aebfd4b7a863",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "JLimperg/msc-thesis-code",
"max_forks_repo_path": "src/Source/Size/Substitution/Canonical.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "104cddc6b65386c7e121c13db417aebfd4b7a863",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "JLimperg/msc-thesis-code",
"max_issues_repo_path": "src/Source/Size/Substitution/Canonical.agda",
"max_line_length": 80,
"max_stars_count": 5,
"max_stars_repo_head_hexsha": "104cddc6b65386c7e121c13db417aebfd4b7a863",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "JLimperg/msc-thesis-code",
"max_stars_repo_path": "src/Source/Size/Substitution/Canonical.agda",
"max_stars_repo_stars_event_max_datetime": "2021-06-26T06:37:31.000Z",
"max_stars_repo_stars_event_min_datetime": "2021-04-13T21:31:17.000Z",
"num_tokens": 3579,
"size": 7724
} |
module Algebra.Module.Normed where
open import Assume using (assume)
open import Algebra.Bundles using (CommutativeRing)
open import Algebra.Module.Bundles using (Module)
open import Level using (_⊔_; suc)
open import Relation.Nullary using (¬_)
open import Relation.Binary using (Rel)
open import Function.Metric using (IsGeneralMetric)
module _
{r ℓr} {CR : CommutativeRing r ℓr}
{m ℓm} (M : Module CR m ℓm)
where
private
module CR = CommutativeRing CR
module M = Module M
module _
{rel} (_≤_ : Rel CR.Carrier rel)
(∥_∥ : M.Carrierᴹ → CR.Carrier)
where
record IsNormedModule : Set (r ⊔ ℓr ⊔ m ⊔ ℓm ⊔ rel) where
open CommutativeRing CR public
open M public
field
triangle-norm : ∀ x y → (∥ x +ᴹ y ∥) ≤ (∥ x ∥ + ∥ y ∥)
homogeneity : ∀ s x → ∥ s *ₗ x ∥ ≈ s * ∥ x ∥
positive-definite : ∀ x → ∥ x ∥ ≈ 0# → x ≈ᴹ 0ᴹ
infixl 6 _-ᴹ_
_-ᴹ_ : Carrierᴹ → Carrierᴹ → Carrierᴹ
x -ᴹ y = x +ᴹ (-ᴹ y)
⟨_,_⟩ : Carrierᴹ → Carrierᴹ → Carrier
⟨ x , y ⟩ = ∥ x -ᴹ y ∥
isGeneralMetric : IsGeneralMetric _≈ᴹ_ _≈_ _≤_ 0# _+_ ⟨_,_⟩
isGeneralMetric = assume
open IsGeneralMetric isGeneralMetric public hiding (refl; reflexive)
module _
{r ℓr} (CR : CommutativeRing r ℓr)
(open CommutativeRing CR using () renaming (Carrier to X))
{rel} (_≤_ : Rel X rel)
m ℓm
where
record NormedModule : Set (suc (r ⊔ ℓr ⊔ m ⊔ ℓm ⊔ rel)) where
module CR = CommutativeRing CR
field
M : Module CR m ℓm
module M = Module M
field
∥_∥ : M.Carrierᴹ → CR.Carrier
isNormedModule : IsNormedModule M _≤_ ∥_∥
open IsNormedModule isNormedModule public
module _
{r ℓr} {CR : CommutativeRing r ℓr}
(open CommutativeRing CR using () renaming (Carrier to X))
{rel} {_≤_ : Rel X rel}
{ma ℓma} (MA : NormedModule CR _≤_ ma ℓma)
{mb ℓmb} (MB : NormedModule CR _≤_ mb ℓmb)
where
private
module CR = CommutativeRing CR
module MA = NormedModule MA
module MB = NormedModule MB
directProduct : NormedModule CR _≤_ (ma ⊔ mb) (ℓma ⊔ ℓmb)
directProduct =
record
{ M = ⟨module⟩ MA.M MB.M
; ∥_∥ = (uncurry CR._+_) ∘ (map MA.∥_∥ MB.∥_∥)
; isNormedModule = assume
}
where
open import Algebra.Module.Construct.DirectProduct
open import Function using (_∘_)
open import Data.Product using (uncurry; map)
module _
{r ℓr} {CR : CommutativeRing r ℓr}
(open CommutativeRing CR using () renaming (Carrier to X))
{rel} {_≤_ : Rel X rel}
(∥_∥ : X → X)
where
tensorUnit : NormedModule CR _≤_ r ℓr
tensorUnit =
record
{ M = ⟨module⟩
; ∥_∥ = ∥_∥
; isNormedModule = assume
}
where open import Algebra.Module.Construct.TensorUnit
module _
{r ℓr} {CR : CommutativeRing r ℓr}
(open CommutativeRing CR using () renaming (Carrier to X))
{rel} {_≤_ : Rel X rel}
where
null : ∀ {c l} → NormedModule CR _≤_ c l
null =
record
{ M = ⟨module⟩
; ∥_∥ = λ _ → 0#
; isNormedModule = assume
}
where
open import Algebra.Module.Construct.Zero
open CommutativeRing CR
-- TODO
-- →NormedModule | {
"alphanum_fraction": 0.6147488875,
"avg_line_length": 24.2,
"ext": "agda",
"hexsha": "733f01fe03b583429974a280d00465efb8a25568",
"lang": "Agda",
"max_forks_count": null,
"max_forks_repo_forks_event_max_datetime": null,
"max_forks_repo_forks_event_min_datetime": null,
"max_forks_repo_head_hexsha": "a193aeebf1326f960975b19d3e31b46fddbbfaa2",
"max_forks_repo_licenses": [
"CC0-1.0"
],
"max_forks_repo_name": "cspollard/reals",
"max_forks_repo_path": "src/Algebra/Module/Normed.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "a193aeebf1326f960975b19d3e31b46fddbbfaa2",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"CC0-1.0"
],
"max_issues_repo_name": "cspollard/reals",
"max_issues_repo_path": "src/Algebra/Module/Normed.agda",
"max_line_length": 74,
"max_stars_count": null,
"max_stars_repo_head_hexsha": "a193aeebf1326f960975b19d3e31b46fddbbfaa2",
"max_stars_repo_licenses": [
"CC0-1.0"
],
"max_stars_repo_name": "cspollard/reals",
"max_stars_repo_path": "src/Algebra/Module/Normed.agda",
"max_stars_repo_stars_event_max_datetime": null,
"max_stars_repo_stars_event_min_datetime": null,
"num_tokens": 1162,
"size": 3146
} |
{-# OPTIONS --cubical --no-exact-split --safe #-}
module Cubical.Data.NatPlusOne.Properties where
open import Cubical.Foundations.Prelude
open import Cubical.Foundations.Isomorphism
open import Cubical.Data.Nat
open import Cubical.Data.NatPlusOne.Base
1+Path : ℕ ≡ ℕ₊₁
1+Path = isoToPath (iso 1+_ -1+_ (λ _ → refl) (λ _ → refl))
| {
"alphanum_fraction": 0.7432024169,
"avg_line_length": 30.0909090909,
"ext": "agda",
"hexsha": "256eb8e7aaadee4f0a4d947da4f32f4a43f11e0a",
"lang": "Agda",
"max_forks_count": null,
"max_forks_repo_forks_event_max_datetime": null,
"max_forks_repo_forks_event_min_datetime": null,
"max_forks_repo_head_hexsha": "c67854d2e11aafa5677e25a09087e176fafd3e43",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "cmester0/cubical",
"max_forks_repo_path": "Cubical/Data/NatPlusOne/Properties.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "c67854d2e11aafa5677e25a09087e176fafd3e43",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "cmester0/cubical",
"max_issues_repo_path": "Cubical/Data/NatPlusOne/Properties.agda",
"max_line_length": 59,
"max_stars_count": 1,
"max_stars_repo_head_hexsha": "c67854d2e11aafa5677e25a09087e176fafd3e43",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "cmester0/cubical",
"max_stars_repo_path": "Cubical/Data/NatPlusOne/Properties.agda",
"max_stars_repo_stars_event_max_datetime": "2020-03-23T23:52:11.000Z",
"max_stars_repo_stars_event_min_datetime": "2020-03-23T23:52:11.000Z",
"num_tokens": 104,
"size": 331
} |
module Common where
open import Level using (Level)
open import Relation.Binary.PropositionalEquality using (_≡_; _≢_; sym; refl)
open import Relation.Nullary.Decidable using (False; toWitnessFalse)
open import Data.Nat using (ℕ)
open import Data.Fin using (Fin; _≟_)
private
variable
n : ℕ
l : Level
A : Set l
x x′ y : A
Label : Set
Label = ℕ
data Action (n : ℕ) : Set where
action : (p q : Fin n) -> p ≢ q -> Label -> Action n
action′ : (p q : Fin n) -> {False (p ≟ q)} -> Label -> Action n
action′ p q {p≢q} l = action p q (toWitnessFalse p≢q) l
¬≡-flip : x ≢ y -> y ≢ x
¬≡-flip x≢y = λ y≡x → x≢y (sym y≡x)
≢-subst-left : x ≢ y -> x ≡ x′ -> x′ ≢ y
≢-subst-left x≢y refl = x≢y
≢-subst-right : y ≢ x -> x ≡ x′ -> y ≢ x′
≢-subst-right y≢x refl = y≢x
| {
"alphanum_fraction": 0.5912596401,
"avg_line_length": 23.5757575758,
"ext": "agda",
"hexsha": "035660b58194fa527c1e47eb69e5734950344316",
"lang": "Agda",
"max_forks_count": null,
"max_forks_repo_forks_event_max_datetime": null,
"max_forks_repo_forks_event_min_datetime": null,
"max_forks_repo_head_hexsha": "3d12eed9d340207d242d70f43c6b34e01d3620de",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "fangyi-zhou/mpst-in-agda",
"max_forks_repo_path": "Common.agda",
"max_issues_count": 1,
"max_issues_repo_head_hexsha": "3d12eed9d340207d242d70f43c6b34e01d3620de",
"max_issues_repo_issues_event_max_datetime": "2021-11-24T11:30:17.000Z",
"max_issues_repo_issues_event_min_datetime": "2021-08-31T10:15:38.000Z",
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "fangyi-zhou/mpst-in-agda",
"max_issues_repo_path": "Common.agda",
"max_line_length": 77,
"max_stars_count": 1,
"max_stars_repo_head_hexsha": "3d12eed9d340207d242d70f43c6b34e01d3620de",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "fangyi-zhou/mpst-in-agda",
"max_stars_repo_path": "Common.agda",
"max_stars_repo_stars_event_max_datetime": "2021-08-14T17:36:53.000Z",
"max_stars_repo_stars_event_min_datetime": "2021-08-14T17:36:53.000Z",
"num_tokens": 312,
"size": 778
} |
module BTA3 where
open import Data.Nat
open import Data.Bool
open import Data.List
-- Binding times
data BT : Set where
S : BT
D : BT
-- defining a data type [BT],where two members are
-- [S] standing for "static" and [D] standing for dynamic.
-- ``subsumption'' binding times; static can be treated as dynamic,
-- but not vice versa
_≼_ : BT → BT → Bool
_≼_ D S = false
_≼_ _ _ = true
-- note that the above function can also be specified as follows,
-- _≼_ : BT → BT → Bool
-- D ≼ S = false
-- _ ≼ _ = true
-- note that the function [≼] specifies that a "static",S, can be treated
-- as a "dynamic",D, and not the other way round
-- since in Agda, pattern matching is conducted in a sequencial fashion,
-- the above specification makes sure that it returns [false] when the
-- first argument is [D] and the second [S] and returns [true] in all
-- the other three cases.
-- BEGIN: stuff that is also in the standard library
-- Standard propositional equality, see also Relation.Binary.PropositionalEquality
data _==_ {A : Set} (x : A) : A → Set where
refl : x == x
-- [_==_] defines an equality proposition
-- it takes two identical elements of one type as arguments and gives one
-- evidence,[refl],for the proposition
-- subst lemma
subst : {A B : Set}{x x' : A} {C : A → B} → x == x' → C x == C x'
subst{A}{B}{x}{.x} refl = refl
-- or being defined in the following manner...
-- my_subst : {A B : Set}{x x' : A}{C : A → B} → x == x' → C x == C x'
-- my_subst refl = refl
-- the above function further helps to construct evidence for equality
-- proposition
-- it says that if two elements are identical then two new elements obtained
-- by applying the former to a function should also be identical
record True : Set where
data False : Set where
-- note that the above is regarding two simple proposition [True] and [False]
-- regarding [True],
-- it is defined as empty record with a single element of type [True],[record{}]
-- the trick here is that the type checker knows this and fills in any implicit
-- arguments of [True] with this element
-- another way of defining [True] as follows,
-- record True : Set where
-- trivial : True
-- trivial = _
-- regarding [False],
-- it is defined as a proposition without any evidence corresponding well to
-- what a [False] proposition really means
isTrue : Bool → Set
isTrue true = True
isTrue false = False
-- note the isTrue b,given b as boolean, is the type of proof that b is equal to
-- true since if it is the case, [isTrue b] returns type [True] where its
-- evidence is automatically filled in by the type checker while if it is not
-- the case there is no way to supply for the evidence due to the way how
-- [false] is constructed
-- END standard library
----------------------
-- Sublists
----------------------
data _cx-≤_ {A : Set} : List A → List A → Set where
cxle-eq : (l : List A) → l cx-≤ l
cxle-lt : ∀ {l₁ l₂} x → l₁ cx-≤ l₂ → l₁ cx-≤ (x ∷ l₂)
lem-cx-≤-trans : {A : Set} → {l₁ : List A} {l₂ : List A} {l₃ : List A} →
l₁ cx-≤ l₂ → l₂ cx-≤ l₃ → l₁ cx-≤ l₃
lem-cx-≤-trans le1 (cxle-eq l) = le1
lem-cx-≤-trans (cxle-eq l) (cxle-lt x e) = cxle-lt x e
lem-cx-≤-trans (cxle-lt x e) (cxle-lt x' e') = cxle-lt x' (lem-cx-≤-trans (cxle-lt x e) e')
_cxle-∷_ : {A : Set} (x : A) (l : List A) → l cx-≤ (x ∷ l)
x cxle-∷ l = cxle-lt x (cxle-eq l)
data _⊆_ {A : Set} : List A → List A → Set where
refl-⊆ : ∀ {l} → l ⊆ l
step-⊆ : ∀ {l} x l₁ l₂ → l ⊆ (l₁ ++ l₂) → l ⊆ (l₁ ++ (x ∷ l₂))
lem-⊆-trans : {A : Set} → {l₁ : List A} {l₂ : List A} {l₃ : List A} →
l₁ ⊆ l₂ → l₂ ⊆ l₃ → l₁ ⊆ l₃
lem-⊆-trans e (refl-⊆ {l}) = e
lem-⊆-trans (refl-⊆ {l}) (step-⊆ x l₁ l₂ e) = step-⊆ x l₁ l₂ e
lem-⊆-trans (step-⊆ x l₁ l₂ e) (step-⊆ x' l₁' l₂' e') = step-⊆ x' l₁' l₂' (lem-⊆-trans (step-⊆ x l₁ l₂ e) e')
-- data _≤1_ {A : Set} : List A → List A → Set where
-- cxle1-eq : (l : List A) → l ≤1 l
-- cxle1-lt : ∀ x (l : List A) → l ≤1 (x ∷ l)
-- data _?∷_ {A : Set} (x : A): List A → Set where
-- yes∷ : (l : List A) → x ?∷ (x ∷ l)
-- no∷ : (l : List A) → x ?∷ l
-- getList : ∀ {A} {x : A} {l : List A} → x ?∷ l → List A
-- getList {x = x} (yes∷ l) = x ∷ l
-- getList {_} {_} {l} (no∷ .l) = l
-- end sublists
-- some lemmas about BT subsumption
lem-bt≼S : {bt : BT} → isTrue (bt ≼ S) → bt == S
lem-bt≼S {S} bt≼S = refl
lem-bt≼S {D} ()
-- which can also be defined as follows,
-- my_lem-bt≼S : {bt : BT} → isTrue (bt ≼ S) → bt == S
-- my_lem-bt≼S {S} _ = refl
-- my_lem-bt≼S {D} ()
lem-D≼bt : {bt : BT} → isTrue (D ≼ bt) → bt == D
lem-D≼bt {S} ()
lem-D≼bt {D} D≼bt = refl
-- Types of the calculus
mutual
-- s ^ BT
data AType : Set where
Ann : BT → SType → AType
-- int | t -> t
data SType : Set where
SInt : SType
SFun : AType → AType → SType
-- aux definitions
ATInt : BT → AType
ATInt bt = Ann bt SInt
ATFun : BT → AType → AType → AType
ATFun bt at1 at2 = Ann bt (SFun at1 at2)
-- note that the above function labels a ground type with annotations [S] or
-- [D],sort of a labelling function
-- projection: get the BT from a type
btof : AType → BT
btof (Ann bt _) = bt
-- a related function which takes an annotated type as argument and returns
-- the annotation of that type
-- "constraint on types: functions have to be at least as dynamic as their component" should be corrected as follows,
-- arguments of function should be as dynamic as the function
data wft : AType → Set where
wf-int : ∀ {bt} → wft (Ann bt SInt)
wf-fun : ∀ {bt at1 at2} → wft at1 → wft at2
→ isTrue (bt ≼ btof at1) → isTrue (bt ≼ btof at2) → wft (Ann bt (SFun at1 at2))
-- the above proposition specifies a set of well-formed [AType]s,
-- any annotated [SInt]s are well-formed, wft (Ann bt SInt) forall bt ∈ BT
-- in case of functional type with annotation, the following two criteria have
-- to be satisfied to be a well form,
-- a. each of its arguments is well-formed
-- b. the annotation of the function and the annotations of its arguments must
-- satisfy [_≼_] relation
-- for instance, the functional type defined above is well-formed while
-- the following is not,
-- Ann D (
-- SFun (Ann S SInt) (Ann D SInt)
-- )
-- in conclusion,for functional type with annotation to be well-formed,
-- each of its arguments annotations has to be [D] when that of the function
-- is [D] while there is no constraint upon the annotations of its arguments
-- when that of the function is [S]
lem-force-bt : ∀ {bt at} → isTrue (bt ≼ btof at) → D == bt → D == btof at
lem-force-bt {S} bt≼at ()
lem-force-bt {D} {Ann S y'} () D=bt
lem-force-bt {D} {Ann D y'} bt≼at D=bt = refl
-- note the above function takes an element[bt] of type [BT] and a type with
-- annotation,
-- if both
-- a. the type is at least as dynamic as [bt]
-- b. [bt == D]
-- then we know that the annotation of the type must be [D] as well
-- and the function in that case returns evidence for that
-- Low-level types; types wihtout binding information
data Type : Set where
TInt : Type
TFun : Type → Type → Type
-- translation from ATypes to low-level types
mutual
strip : AType → Type
strip (Ann _ σ) = strip' σ
strip' : SType → Type
strip' SInt = TInt
strip' (SFun y y') = TFun (strip y) (strip y')
-- note that the above function [strip] converts a type with annotation [AType]
-- to a low-level type [Type],
-- for instance,
-- strip (Ann D SInt)
-- = strip' SInt
-- = TInt
-- strip (Ann S
-- SFun (Ann S SInt) (Ann D SInt)
-- )
-- = strip' (SFun (Ann S SInt) (Ann D SInt))
-- = TFun (strip (Ann S SInt)) (strip (Ann D SInt))
-- = TFun (strip' SInt) (strip' SInt)
-- = TFun TInt TInt^
-- More general purpose definitions (should also be in standard library)
-- list membership
infix 4 _∈_
data _∈_ {A : Set} : A → List A → Set where
hd : ∀ {x xs} → x ∈ (x ∷ xs)
tl : ∀ {x y xs} → x ∈ xs → x ∈ (y ∷ xs)
-- note the above proposition gives us two constructors for getting
-- evidences for an element being a member of one list
-- end general purpose definitions
-- Typing context
Ctx = List Type
--data Exp' (Γ Γ' : Ctx) : Type → Set where
-- EVar' :
-- Typed expression
data Exp (Γ : Ctx) : Type → Set where
-- [EVar] corresponds to the bounded variables in [AExp]
EVar : ∀ {τ} → τ ∈ Γ → Exp Γ τ
EInt : ℕ → Exp Γ TInt
EFun : ∀ {τ₁ τ₂} → Exp (τ₂ ∷ Γ) τ₁ → Exp Γ (TFun τ₂ τ₁)
EApp : ∀ {τ₁ τ₂} → Exp Γ (TFun τ₂ τ₁) → Exp Γ τ₂ → Exp Γ τ₁
-- one additional term,
count_tl : ∀ {A Γ Γ'} {τ : A } → τ ∈ Γ → Γ cx-≤ Γ' → τ ∈ Γ'
count_tl x (cxle-eq Γ) = x
count_tl x (cxle-lt T e) = tl (count_tl x e)
data _cx=≤_ {A : Set} : List A → List A → Set where
cxle-peq : ∀ {l₁ l₂} { x } → l₁ cx-≤ l₂ → (x ∷ l₁) cx=≤ (x ∷ l₂)
cxle-plt : ∀ {l₁ l₂} { x } → l₁ cx=≤ l₂ → (x ∷ l₁) cx=≤ (x ∷ l₂)
count_tl' : ∀ {A Γ Γ'} {τ : A } → τ ∈ Γ → Γ cx=≤ Γ' → τ ∈ Γ'
count_tl' hd (cxle-plt e) = hd
count_tl' hd (cxle-peq e) = hd
count_tl' (tl xid) (cxle-plt e) = tl (count_tl' xid e)
count_tl' (tl xid) (cxle-peq e) = tl (count_tl xid e)
lem-Exp-weakening' : ∀ {τ₂ τ₁ Γ Γ'} → Exp (τ₂ ∷ Γ) τ₁ → (τ₂ ∷ Γ) cx=≤ (τ₂ ∷ Γ') → Exp (τ₂ ∷ Γ') τ₁
lem-Exp-weakening' (EVar x) e = EVar (count_tl' x e)
lem-Exp-weakening' (EInt n) e = EInt n
lem-Exp-weakening' (EFun t) e = EFun (lem-Exp-weakening' t (cxle-plt e))
lem-Exp-weakening' (EApp t1 t2) e = EApp (lem-Exp-weakening' t1 e) (lem-Exp-weakening' t2 e)
lem-Exp-weakening : ∀ {τ Γ Γ'} → Exp Γ τ → Γ cx-≤ Γ' → Exp Γ' τ
lem-Exp-weakening t (cxle-eq Γ) = t
lem-Exp-weakening (EInt n) e = EInt n
lem-Exp-weakening (EVar x) e = EVar (count_tl x e)
lem-Exp-weakening (EFun t) (cxle-lt T e) = EFun (lem-Exp-weakening' t (cxle-peq (cxle-lt T e)))
lem-Exp-weakening (EApp t1 t2) e = EApp (lem-Exp-weakening t1 e) (lem-Exp-weakening t2 e)
-- typed annotated expressions
ACtx = List AType
data AExp (Δ : ACtx) : AType → Set where
AVar : ∀ {α} → α ∈ Δ → AExp Δ α
AInt : (bt : BT) → ℕ → AExp Δ (ATInt bt)
AFun : ∀ {α₁ α₂} (bt : BT) → wft (ATFun bt α₂ α₁) → AExp (α₂ ∷ Δ) α₁ → AExp Δ (ATFun bt α₂ α₁)
AApp : ∀ {α₁ α₂} (bt : BT) → wft (ATFun bt α₂ α₁) → AExp Δ (ATFun bt α₂ α₁) → AExp Δ α₂ → AExp Δ α₁
-- stripping of contexts
residual : ACtx → Ctx
residual [] = []
residual (Ann S _ ∷ xs) = residual xs
residual (Ann D σ ∷ xs) = strip' σ ∷ residual xs
-- ``semantic domain'' for partially evaluated AExp-terms:
-- - AExp-terms of dynamic type evaluate to Exp-terms
-- - AExp-terms of static type evaluate to agda terms, where SFun
-- are functions and SInt are natural numbers
mutual
impTA : Ctx → AType → Set
impTA Γ (Ann S σ) = impTA' Γ σ
impTA Γ (Ann D σ) = Exp Γ (strip' σ)
impTA' : Ctx → SType → Set
impTA' Γ SInt = ℕ
-- impTA' Γ (SFun y y') = impTA Γ y → impTA Γ y'
impTA' Γ (SFun y y') = ∀ {Γ'} → Γ cx-≤ Γ' → impTA Γ' y → impTA Γ' y'
lem-impTA-weakening : ∀ {α Γ Γ'} →
impTA Γ α →
Γ cx-≤ Γ' →
impTA Γ' α
lem-impTA-weakening {Ann S SInt} v _ = v
lem-impTA-weakening {Ann S (SFun x x₁)} f prf = λ prf' → f (lem-cx-≤-trans prf prf')
lem-impTA-weakening {Ann D x₁} v prf = lem-Exp-weakening v prf
-- mutual
-- impTA-try : Ctx → AType → Set
-- impTA-try Γ (Ann S σ) = impTA-try' Γ σ
-- impTA-try Γ (Ann D σ) = Exp Γ (strip' σ)
-- impTA-try' : Ctx → SType → Set
-- impTA-try' Γ SInt = ℕ
-- impTA-try' Γ (SFun y y') = impTA-try Γ y → impTA-try Γ y'
-- lem-impTA-try-weakening : ∀ {α Γ Γ'} →
-- impTA-try Γ α →
-- Γ cx-≤ Γ' →
-- impTA-try Γ' α
-- lem-impTA-try-weakening {Ann S SInt} v _ = v
-- lem-impTA-try-weakening {Ann S (SFun α x₁)} {Γ} {Γ'} f prf = {! λ (v : impTA-try Γ' α) → f v!}
-- lem-impTA-try-weakening {Ann D x₁} v prf = lem-Exp-weakening v prf
data AEnv : Ctx → ACtx → Set where
env[] : ∀ {Γ} → AEnv Γ []
envS:: : ∀ {Γ Δ} {α} →
impTA Γ α →
AEnv Γ Δ →
AEnv Γ (α ∷ Δ)
envD:: : ∀ {Γ Δ} →
(σ : SType) →
impTA (strip' σ ∷ Γ) (Ann D σ) →
AEnv Γ Δ →
AEnv (strip' σ ∷ Γ) (Ann D σ ∷ Δ)
lem-AEnv-weakening : ∀ {Γ Γ' Δ} → AEnv Γ Δ → Γ cx-≤ Γ' → AEnv Γ' Δ
lem-AEnv-weakening env[] prf = env[]
lem-AEnv-weakening (envS:: {α = α} x env) prf = envS:: (lem-impTA-weakening {α} x prf) (lem-AEnv-weakening env prf)
lem-AEnv-weakening (envD:: {Γ} σ x env) prf = envS:: (lem-impTA-weakening {Ann D σ} x prf) (lem-AEnv-weakening env (lem-cx-≤-trans (cxle-lt (strip' σ) (cxle-eq Γ)) prf)) -- non-primitive recursion... this should be fixable by extending Γ in the middle, rather than in the end
lookup : ∀ {Γ Δ α} → AEnv Γ Δ → (o : α ∈ Δ ) → impTA Γ α
lookup env[] ()
lookup (envS:: x env) hd = x
lookup (envS:: x env) (tl idx) = lookup env idx
lookup (envD:: σ x env) hd = x
lookup {α = α} (envD:: {Γ} σ x env) (tl idx) = lem-impTA-weakening {α} (lookup env idx) (strip' σ cxle-∷ Γ)
data IsDynamic : AType → Set where
is-dyn : ∀ σ → IsDynamic (Ann D σ)
lem-IsDynamic-by-wf : ∀ α → isTrue (D ≼ btof α) → IsDynamic α
lem-IsDynamic-by-wf (Ann S σ) ()
lem-IsDynamic-by-wf (Ann D σ) _ = is-dyn σ
-- TODO: Do we need additional assurance in the type signature (or as
-- an aux. lemma) that Γ is the residue of Δ?
pe : ∀ {Δ Γ α} → AEnv Γ Δ → AExp Δ α → impTA Γ α
pe env (AVar idx) = lookup env idx
pe env (AInt S i) = i
pe env (AInt D i) = EInt i
pe {Γ = Γ} env (AFun {α₁} {α₂} S prf exp) = λ {Γ'} (prf₁ : Γ cx-≤ Γ') (v : impTA Γ' α₂) →
pe (envS:: v (lem-AEnv-weakening env prf₁)) exp
pe env (AFun {α₁} {α₂} D (wf-fun _ _ prf-2 prf-1) e)
with lem-IsDynamic-by-wf α₁ prf-1 | lem-IsDynamic-by-wf α₂ prf-2
pe {Γ = Γ} env (AFun {.(Ann D σ₁)} {.(Ann D σ₂)} D (wf-fun _ _ prf-1 prf-2) e)
| is-dyn σ₁ | is-dyn σ₂ =
EFun (pe (envD:: σ₂ (EVar hd) env) e)
pe {Γ = Γ} env (AApp S _ f e) = (pe env f (cxle-eq Γ)) (pe env e)
pe env (AApp {α₁} {α₂} D (wf-fun _ _ prf-2 prf-1) f e)
with lem-IsDynamic-by-wf α₁ prf-1 | lem-IsDynamic-by-wf α₂ prf-2
pe env (AApp {.(Ann D σ₁)}{.(Ann D σ₂)} D (wf-fun _ _ prf-2 prf-1) f e)
| is-dyn σ₁ | is-dyn σ₂ =
EApp (pe env f) (pe env e) -- construct an Exp-application using the proof that argument and results are dynamic and thus pe yields Exp-terms for them
| {
"alphanum_fraction": 0.5958683473,
"avg_line_length": 34.8292682927,
"ext": "agda",
"hexsha": "3365b313affa2cd7bebe6bb1a7dcaf2b8dd88f56",
"lang": "Agda",
"max_forks_count": 1,
"max_forks_repo_forks_event_max_datetime": "2019-10-15T09:01:37.000Z",
"max_forks_repo_forks_event_min_datetime": "2019-10-15T09:01:37.000Z",
"max_forks_repo_head_hexsha": "ef878f7fa5afa51fb7a14cd8f7f75da0af1b9deb",
"max_forks_repo_licenses": [
"BSD-3-Clause"
],
"max_forks_repo_name": "luminousfennell/polybta",
"max_forks_repo_path": "BTA3.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "ef878f7fa5afa51fb7a14cd8f7f75da0af1b9deb",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"BSD-3-Clause"
],
"max_issues_repo_name": "luminousfennell/polybta",
"max_issues_repo_path": "BTA3.agda",
"max_line_length": 276,
"max_stars_count": 1,
"max_stars_repo_head_hexsha": "ef878f7fa5afa51fb7a14cd8f7f75da0af1b9deb",
"max_stars_repo_licenses": [
"BSD-3-Clause"
],
"max_stars_repo_name": "luminousfennell/polybta",
"max_stars_repo_path": "BTA3.agda",
"max_stars_repo_stars_event_max_datetime": "2019-10-15T04:35:29.000Z",
"max_stars_repo_stars_event_min_datetime": "2019-10-15T04:35:29.000Z",
"num_tokens": 5405,
"size": 14280
} |
{-# OPTIONS --safe #-}
module Cubical.Algebra.Module where
open import Cubical.Algebra.Module.Base public
| {
"alphanum_fraction": 0.7663551402,
"avg_line_length": 21.4,
"ext": "agda",
"hexsha": "6528a163e8d6f5eb599e97412f92cfd63b81d77c",
"lang": "Agda",
"max_forks_count": 134,
"max_forks_repo_forks_event_max_datetime": "2022-03-23T16:22:13.000Z",
"max_forks_repo_forks_event_min_datetime": "2018-11-16T06:11:03.000Z",
"max_forks_repo_head_hexsha": "53e159ec2e43d981b8fcb199e9db788e006af237",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "marcinjangrzybowski/cubical",
"max_forks_repo_path": "Cubical/Algebra/Module.agda",
"max_issues_count": 584,
"max_issues_repo_head_hexsha": "53e159ec2e43d981b8fcb199e9db788e006af237",
"max_issues_repo_issues_event_max_datetime": "2022-03-30T12:09:17.000Z",
"max_issues_repo_issues_event_min_datetime": "2018-10-15T09:49:02.000Z",
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "marcinjangrzybowski/cubical",
"max_issues_repo_path": "Cubical/Algebra/Module.agda",
"max_line_length": 46,
"max_stars_count": 301,
"max_stars_repo_head_hexsha": "53e159ec2e43d981b8fcb199e9db788e006af237",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "marcinjangrzybowski/cubical",
"max_stars_repo_path": "Cubical/Algebra/Module.agda",
"max_stars_repo_stars_event_max_datetime": "2022-03-24T02:10:47.000Z",
"max_stars_repo_stars_event_min_datetime": "2018-10-17T18:00:24.000Z",
"num_tokens": 23,
"size": 107
} |
module RMonads.CatofRMonads where
open import Categories
open import Functors
open import RMonads
open import RMonads.RMonadMorphs
CatofRMonads : ∀{a b c d}{C : Cat {a}{b}}{D : Cat {c}{d}}(J : Fun C D) → Cat
CatofRMonads J = record
{ Obj = RMonad J
; Hom = RMonadMorph
; iden = IdRMonadMorph _
; comp = CompRMonadMorph
; idl = idl _
; idr = idr _
; ass = λ{_ _ _ _ f g h} → ass f g h
}
| {
"alphanum_fraction": 0.4952741021,
"avg_line_length": 29.3888888889,
"ext": "agda",
"hexsha": "e57da8f51f53ee9f88d552c618b8e798327b2dc0",
"lang": "Agda",
"max_forks_count": 1,
"max_forks_repo_forks_event_max_datetime": "2019-11-04T21:33:13.000Z",
"max_forks_repo_forks_event_min_datetime": "2019-11-04T21:33:13.000Z",
"max_forks_repo_head_hexsha": "74707d3538bf494f4bd30263d2f5515a84733865",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "jmchapman/Relative-Monads",
"max_forks_repo_path": "RMonads/CatofRMonads.agda",
"max_issues_count": 3,
"max_issues_repo_head_hexsha": "74707d3538bf494f4bd30263d2f5515a84733865",
"max_issues_repo_issues_event_max_datetime": "2019-05-29T09:50:26.000Z",
"max_issues_repo_issues_event_min_datetime": "2019-01-13T13:12:33.000Z",
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "jmchapman/Relative-Monads",
"max_issues_repo_path": "RMonads/CatofRMonads.agda",
"max_line_length": 76,
"max_stars_count": 21,
"max_stars_repo_head_hexsha": "74707d3538bf494f4bd30263d2f5515a84733865",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "jmchapman/Relative-Monads",
"max_stars_repo_path": "RMonads/CatofRMonads.agda",
"max_stars_repo_stars_event_max_datetime": "2021-02-13T18:02:18.000Z",
"max_stars_repo_stars_event_min_datetime": "2015-07-30T01:25:12.000Z",
"num_tokens": 167,
"size": 529
} |
-- Andreas, 2014-10-09, issue reported by jesper.cockx
open import Common.Product
pattern foo x = x , x
-- Should complain about non-linearity.
test : {A : Set} → A × A → A
test (foo x) = x
| {
"alphanum_fraction": 0.6632124352,
"avg_line_length": 19.3,
"ext": "agda",
"hexsha": "1e8ea17b7d0cf6ee69d78785268408233262d62b",
"lang": "Agda",
"max_forks_count": 371,
"max_forks_repo_forks_event_max_datetime": "2022-03-30T19:00:30.000Z",
"max_forks_repo_forks_event_min_datetime": "2015-01-03T14:04:08.000Z",
"max_forks_repo_head_hexsha": "7f58030124fa99dfbf8db376659416f3ad8384de",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "cruhland/agda",
"max_forks_repo_path": "test/Fail/Issue1295.agda",
"max_issues_count": 4066,
"max_issues_repo_head_hexsha": "7f58030124fa99dfbf8db376659416f3ad8384de",
"max_issues_repo_issues_event_max_datetime": "2022-03-31T21:14:49.000Z",
"max_issues_repo_issues_event_min_datetime": "2015-01-10T11:24:51.000Z",
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "cruhland/agda",
"max_issues_repo_path": "test/Fail/Issue1295.agda",
"max_line_length": 54,
"max_stars_count": 1989,
"max_stars_repo_head_hexsha": "7f58030124fa99dfbf8db376659416f3ad8384de",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "cruhland/agda",
"max_stars_repo_path": "test/Fail/Issue1295.agda",
"max_stars_repo_stars_event_max_datetime": "2022-03-30T18:20:48.000Z",
"max_stars_repo_stars_event_min_datetime": "2015-01-09T23:51:16.000Z",
"num_tokens": 63,
"size": 193
} |
{-# OPTIONS --safe #-}
module Cubical.HITs.FreeComMonoids.Properties where
open import Cubical.Foundations.Everything hiding (assoc; ⟨_⟩)
open import Cubical.Data.Nat hiding (_·_ ; _^_)
open import Cubical.HITs.FreeComMonoids.Base as FCM
open import Cubical.HITs.AssocList as AL
private variable
ℓ : Level
A : Type ℓ
multi-· : A → ℕ → FreeComMonoid A → FreeComMonoid A
multi-· x zero xs = xs
multi-· x (suc n) xs = ⟦ x ⟧ · multi-· x n xs
_^_ : A → ℕ → FreeComMonoid A
x ^ n = multi-· x n ε
^+≡ : ∀ (p : A) m n → ((p ^ m) · (p ^ n)) ≡ (p ^ (m + n))
^+≡ p zero n = identityₗ _
^+≡ p (suc m) n = sym (assoc _ _ _) ∙ cong (_ ·_) (^+≡ _ _ _)
AL→FCM : AssocList A → FreeComMonoid A
AL→FCM = AL.Rec.f trunc ε (λ a n p → (a ^ n) · p)
per* agg* (const identityₗ)
where
per* : ∀ x y (mon : FreeComMonoid A) →
((⟦ x ⟧ · ε) · ((⟦ y ⟧ · ε) · mon)) ≡
((⟦ y ⟧ · ε) · ((⟦ x ⟧ · ε) · mon))
per* x y mon =
(⟦ x ⟧ · ε) · ((⟦ y ⟧ · ε) · mon)
≡⟨ assoc _ _ _ ⟩
((⟦ x ⟧ · ε) · (⟦ y ⟧ · ε)) · mon
≡⟨ cong (_· mon) (comm _ _) ⟩
(((⟦ y ⟧ · ε) · (⟦ x ⟧ · ε)) · mon)
≡⟨ sym (assoc _ _ _) ⟩
((⟦ y ⟧ · ε) · ((⟦ x ⟧ · ε) · mon)) ∎
agg* : ∀ a m n mon →
((a ^ m) · ((a ^ n) · mon)) ≡ ((a ^ (m + n)) · mon)
agg* a m n mon =
((a ^ m) · ((a ^ n) · mon))
≡⟨ assoc _ _ _ ⟩
(((a ^ m) · (a ^ n)) · mon)
≡⟨ cong (_· _) (^+≡ _ _ _) ⟩
((a ^ (m + n)) · mon) ∎
FCM→AL : FreeComMonoid A → AssocList A
FCM→AL = FCM.Rec.f trunc ⟨_⟩ ⟨⟩ _++_ comm-++ unitr-++ (λ _ → refl) assoc-++
^-id : (x : A) (m : ℕ) (u : FreeComMonoid A)
→ FCM→AL ((x ^ m) · u) ≡ ⟨ x , m ⟩∷ FCM→AL u
^-id x zero u = cong FCM→AL (identityₗ u) ∙ sym (del _ _)
^-id x (suc m) u =
FCM→AL ((⟦ x ⟧ · (x ^ m)) · u)
≡⟨ cong ⟨ x , 1 ⟩∷_ (^-id x m u) ⟩
⟨ x , 1 ⟩∷ ⟨ x , m ⟩∷ FCM→AL u
≡⟨ agg _ _ _ _ ⟩
⟨ x , suc m ⟩∷ FCM→AL u ∎
++-· : (x y : AssocList A)
→ AL→FCM (x ++ y) ≡ AL→FCM x · AL→FCM y
++-· = AL.ElimProp.f
(isPropΠ (λ _ → trunc _ _))
(λ _ → sym (identityₗ _))
λ x n {xs} p ys →
AL→FCM (((⟨ x , n ⟩∷ ⟨⟩) ++ xs) ++ ys)
≡⟨ cong AL→FCM (cong (_++ ys) (comm-++ (⟨ x , n ⟩∷ ⟨⟩) xs) ∙ sym (assoc-++ xs _ ys)) ⟩
AL→FCM (xs ++ (⟨ x , n ⟩∷ ys))
≡⟨ p _ ⟩
(AL→FCM xs · ((x ^ n) · AL→FCM ys))
≡⟨ assoc (AL→FCM xs) _ _ ⟩
((AL→FCM xs · (x ^ n)) · AL→FCM ys)
≡⟨ cong (_· AL→FCM ys) (comm _ _) ⟩
((x ^ n) · AL→FCM xs) · AL→FCM ys ∎
AL→FCM∘FCM→AL≡id : section {A = AssocList A} AL→FCM FCM→AL
AL→FCM∘FCM→AL≡id = FCM.ElimProp.f (trunc _ _) (λ x → identityᵣ _ ∙ identityᵣ _) refl
λ {x y} p q → ++-· (FCM→AL x) (FCM→AL y) ∙ cong₂ _·_ p q
FCM→AL∘AL→FCM≡id : retract {A = AssocList A} AL→FCM FCM→AL
FCM→AL∘AL→FCM≡id = AL.ElimProp.f (trunc _ _) refl
λ x n {xs} p → ^-id x n (AL→FCM xs) ∙ cong (⟨ _ , _ ⟩∷_) p
AssocList≃FreeComMonoid : AssocList A ≃ FreeComMonoid A
AssocList≃FreeComMonoid = isoToEquiv (iso AL→FCM FCM→AL AL→FCM∘FCM→AL≡id FCM→AL∘AL→FCM≡id)
AssocList≡FreeComMonoid : AssocList A ≡ FreeComMonoid A
AssocList≡FreeComMonoid = ua AssocList≃FreeComMonoid
| {
"alphanum_fraction": 0.4998331665,
"avg_line_length": 31.8829787234,
"ext": "agda",
"hexsha": "588aaaa9a4f28dcc064765cf47d93aceff3b6e6d",
"lang": "Agda",
"max_forks_count": null,
"max_forks_repo_forks_event_max_datetime": null,
"max_forks_repo_forks_event_min_datetime": null,
"max_forks_repo_head_hexsha": "1b9c97a2140fe96fe636f4c66beedfd7b8096e8f",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "howsiyu/cubical",
"max_forks_repo_path": "Cubical/HITs/FreeComMonoids/Properties.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "1b9c97a2140fe96fe636f4c66beedfd7b8096e8f",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "howsiyu/cubical",
"max_issues_repo_path": "Cubical/HITs/FreeComMonoids/Properties.agda",
"max_line_length": 90,
"max_stars_count": null,
"max_stars_repo_head_hexsha": "1b9c97a2140fe96fe636f4c66beedfd7b8096e8f",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "howsiyu/cubical",
"max_stars_repo_path": "Cubical/HITs/FreeComMonoids/Properties.agda",
"max_stars_repo_stars_event_max_datetime": null,
"max_stars_repo_stars_event_min_datetime": null,
"num_tokens": 1480,
"size": 2997
} |
module CoInf where
open import Coinduction
-- Check that ∞ can be used as an "expression".
test : Set → Set
test = ∞
| {
"alphanum_fraction": 0.6974789916,
"avg_line_length": 14.875,
"ext": "agda",
"hexsha": "a40eca0bdd6aa197c11a0585f7f1a433447023d2",
"lang": "Agda",
"max_forks_count": 1,
"max_forks_repo_forks_event_max_datetime": "2019-03-05T20:02:38.000Z",
"max_forks_repo_forks_event_min_datetime": "2019-03-05T20:02:38.000Z",
"max_forks_repo_head_hexsha": "56928ff709dcb931cb9a48c4790e5ed3739e3032",
"max_forks_repo_licenses": [
"BSD-3-Clause"
],
"max_forks_repo_name": "andersk/agda",
"max_forks_repo_path": "test/LibSucceed/CoInf.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "56928ff709dcb931cb9a48c4790e5ed3739e3032",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"BSD-3-Clause"
],
"max_issues_repo_name": "andersk/agda",
"max_issues_repo_path": "test/LibSucceed/CoInf.agda",
"max_line_length": 47,
"max_stars_count": 3,
"max_stars_repo_head_hexsha": "04941fb75be06039b0085ab047117625294cbc99",
"max_stars_repo_licenses": [
"BSD-3-Clause"
],
"max_stars_repo_name": "andreasabel/agda-with-old-branches",
"max_stars_repo_path": "test/LibSucceed/CoInf.agda",
"max_stars_repo_stars_event_max_datetime": "2015-12-07T20:14:00.000Z",
"max_stars_repo_stars_event_min_datetime": "2015-03-28T14:51:03.000Z",
"num_tokens": 35,
"size": 119
} |
module Structure.Operator.Monoid.Proofs where
import Lvl
open import Logic
open import Logic.Propositional
open import Logic.Predicate
open import Structure.Setoid
open import Structure.Operator.Monoid
open import Structure.Operator.Properties
open import Structure.Operator.Proofs
open import Type
| {
"alphanum_fraction": 0.8431372549,
"avg_line_length": 23.5384615385,
"ext": "agda",
"hexsha": "9daed68f3e6b81a11b8e9b20b2ba30609941f785",
"lang": "Agda",
"max_forks_count": null,
"max_forks_repo_forks_event_max_datetime": null,
"max_forks_repo_forks_event_min_datetime": null,
"max_forks_repo_head_hexsha": "70f4fba849f2fd779c5aaa5af122ccb6a5b271ba",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "Lolirofle/stuff-in-agda",
"max_forks_repo_path": "Structure/Operator/Monoid/Proofs.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "70f4fba849f2fd779c5aaa5af122ccb6a5b271ba",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "Lolirofle/stuff-in-agda",
"max_issues_repo_path": "Structure/Operator/Monoid/Proofs.agda",
"max_line_length": 45,
"max_stars_count": 6,
"max_stars_repo_head_hexsha": "70f4fba849f2fd779c5aaa5af122ccb6a5b271ba",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "Lolirofle/stuff-in-agda",
"max_stars_repo_path": "Structure/Operator/Monoid/Proofs.agda",
"max_stars_repo_stars_event_max_datetime": "2022-02-05T06:53:22.000Z",
"max_stars_repo_stars_event_min_datetime": "2020-04-07T17:58:13.000Z",
"num_tokens": 60,
"size": 306
} |
{-# OPTIONS --without-K --safe #-}
module Categories.Bicategory.Extras where
open import Data.Product using (_,_)
open import Categories.Bicategory using (Bicategory)
open import Categories.Functor using (Functor)
open import Categories.Functor.Bifunctor using (appʳ; appˡ)
open import Categories.Functor.Bifunctor.Properties using ([_]-commute)
open import Categories.NaturalTransformation.NaturalIsomorphism using (NaturalIsomorphism)
import Categories.Morphism as Mor
import Categories.Morphism.Reasoning as MR
module Extras {o ℓ e t} (Bicat : Bicategory o ℓ e t) where
open Bicategory Bicat
private
variable
A B C D : Obj
f g h i : A ⇒₁ B
α β γ : f ⇒₂ g
module ⊚ {A B C} = Functor (⊚ {A} {B} {C})
module ⊚-assoc {A B C D} = NaturalIsomorphism (⊚-assoc {A} {B} {C} {D})
module unitˡ {A B} = NaturalIsomorphism (unitˡ {A} {B})
module unitʳ {A B} = NaturalIsomorphism (unitʳ {A} {B})
module id {A} = Functor (id {A})
unitorˡ : {A B : Obj} {f : A ⇒₁ B} → Mor._≅_ (hom A B) (id₁ ∘ₕ f) f
unitorˡ {_} {_} {f} = record
{ from = unitˡ.⇒.η (_ , f)
; to = unitˡ.⇐.η (_ , f)
; iso = unitˡ.iso (_ , f)
}
module unitorˡ {A B f} = Mor._≅_ (unitorˡ {A} {B} {f})
unitorʳ : {A B : Obj} {f : A ⇒₁ B} → Mor._≅_ (hom A B) (f ∘ₕ id₁) f
unitorʳ {_} {_} {f} = record
{ from = unitʳ.⇒.η (f , _)
; to = unitʳ.⇐.η (f , _)
; iso = unitʳ.iso (f , _)
}
module unitorʳ {A B f} = Mor._≅_ (unitorʳ {A} {B} {f})
associator : {A B C D : Obj} {f : D ⇒₁ B} {g : C ⇒₁ D} {h : A ⇒₁ C} → Mor._≅_ (hom A B) ((f ∘ₕ g) ∘ₕ h) (f ∘ₕ g ∘ₕ h)
associator {_} {_} {_} {_} {f} {g} {h} = record
{ from = ⊚-assoc.⇒.η ((f , g) , h)
; to = ⊚-assoc.⇐.η ((f , g) , h)
; iso = ⊚-assoc.iso ((f , g) , h)
}
module associator {A B C D} {f : C ⇒₁ B} {g : D ⇒₁ C} {h} = Mor._≅_ (associator {A = A} {B = B} {f = f} {g = g} {h = h})
-⊚_ : C ⇒₁ A → Functor (hom A B) (hom C B)
-⊚_ = appʳ ⊚
_⊚- : B ⇒₁ C → Functor (hom A B) (hom A C)
_⊚- = appˡ ⊚
identity₂ˡ : id₂ ∘ᵥ α ≈ α
identity₂ˡ = hom.identityˡ
identity₂ʳ : α ∘ᵥ id₂ ≈ α
identity₂ʳ = hom.identityʳ
assoc₂ : (α ∘ᵥ β) ∘ᵥ γ ≈ α ∘ᵥ β ∘ᵥ γ
assoc₂ = hom.assoc
id₂◁ : id₂ {f = g} ◁ f ≈ id₂
id₂◁ = ⊚.identity
▷id₂ : f ▷ id₂ {f = g} ≈ id₂
▷id₂ = ⊚.identity
open hom.HomReasoning
open hom.Equiv
private
module MR′ {A} {B} where
open MR (hom A B) using (conjugate-to) public
open Mor (hom A B) using (module ≅) public
open MR′
∘ᵥ-distr-◁ : (α ◁ f) ∘ᵥ (β ◁ f) ≈ (α ∘ᵥ β) ◁ f
∘ᵥ-distr-◁ {f = f} = ⟺ (Functor.homomorphism (-⊚ f))
∘ᵥ-distr-▷ : (f ▷ α) ∘ᵥ (f ▷ β) ≈ f ▷ (α ∘ᵥ β)
∘ᵥ-distr-▷ {f = f} = ⟺ (Functor.homomorphism (f ⊚-))
ρ-∘ᵥ-▷ : unitorˡ.from ∘ᵥ (id₁ ▷ α) ≈ α ∘ᵥ unitorˡ.from
ρ-∘ᵥ-▷ {α = α} = begin
unitorˡ.from ∘ᵥ (id₁ ▷ α) ≈˘⟨ hom.∘-resp-≈ʳ (⊚.F-resp-≈ (id.identity , refl)) ⟩
unitorˡ.from ∘ᵥ id.F₁ _ ⊚₁ α ≈⟨ unitˡ.⇒.commute (_ , α) ⟩
α ∘ᵥ unitorˡ.from ∎
▷-∘ᵥ-ρ⁻¹ : (id₁ ▷ α) ∘ᵥ unitorˡ.to ≈ unitorˡ.to ∘ᵥ α
▷-∘ᵥ-ρ⁻¹ = conjugate-to (≅.sym unitorˡ) (≅.sym unitorˡ) ρ-∘ᵥ-▷
λ-∘ᵥ-◁ : unitorʳ.from ∘ᵥ (α ◁ id₁) ≈ α ∘ᵥ unitorʳ.from
λ-∘ᵥ-◁ {α = α} = begin
unitorʳ.from ∘ᵥ (α ◁ id₁) ≈˘⟨ hom.∘-resp-≈ʳ (⊚.F-resp-≈ (refl , id.identity)) ⟩
unitorʳ.from ∘ᵥ (α ⊚₁ id.F₁ _) ≈⟨ unitʳ.⇒.commute (α , _) ⟩
α ∘ᵥ unitorʳ.from ∎
◁-∘ᵥ-λ⁻¹ : (α ◁ id₁) ∘ᵥ unitorʳ.to ≈ unitorʳ.to ∘ᵥ α
◁-∘ᵥ-λ⁻¹ = conjugate-to (≅.sym unitorʳ) (≅.sym unitorʳ) λ-∘ᵥ-◁
assoc⁻¹-◁-∘ₕ : associator.to ∘ᵥ (α ◁ (g ∘ₕ f)) ≈ ((α ◁ g) ◁ f) ∘ᵥ associator.to
assoc⁻¹-◁-∘ₕ {α = α} {g = g} {f = f} = begin
associator.to ∘ᵥ (α ◁ (g ∘ₕ f)) ≈˘⟨ hom.∘-resp-≈ʳ (⊚.F-resp-≈ (refl , ⊚.identity)) ⟩
associator.to ∘ᵥ (α ⊚₁ id₂ ⊚₁ id₂) ≈⟨ ⊚-assoc.⇐.commute ((α , id₂) , id₂) ⟩
((α ◁ g) ◁ f) ∘ᵥ associator.to ∎
assoc⁻¹-▷-◁ : associator.to ∘ᵥ (f ▷ (α ◁ g)) ≈ ((f ▷ α) ◁ g) ∘ᵥ associator.to
assoc⁻¹-▷-◁ {f = f} {α = α} {g = g} = ⊚-assoc.⇐.commute ((id₂ , α) , id₂)
assoc⁻¹-▷-∘ₕ : associator.to ∘ᵥ (g ▷ (f ▷ α)) ≈ ((g ∘ₕ f) ▷ α) ∘ᵥ associator.to
assoc⁻¹-▷-∘ₕ {g = g} {f = f} {α = α} = begin
associator.to ∘ᵥ (g ▷ (f ▷ α)) ≈⟨ ⊚-assoc.⇐.commute ((id₂ , id₂) , α) ⟩
((id₂ ⊚₁ id₂) ⊚₁ α) ∘ᵥ associator.to ≈⟨ hom.∘-resp-≈ˡ (⊚.F-resp-≈ (⊚.identity , refl)) ⟩
((g ∘ₕ f) ▷ α) ∘ᵥ associator.to ∎
◁-▷-exchg : ∀ {α : f ⇒₂ g} {β : h ⇒₂ i} → (i ▷ α) ∘ᵥ (β ◁ f) ≈ (β ◁ g) ∘ᵥ (h ▷ α)
◁-▷-exchg = [ ⊚ ]-commute
| {
"alphanum_fraction": 0.5086975914,
"avg_line_length": 35.3070866142,
"ext": "agda",
"hexsha": "90d03553735e9308328febeea74575c4739ae415",
"lang": "Agda",
"max_forks_count": 1,
"max_forks_repo_forks_event_max_datetime": "2021-11-04T06:54:45.000Z",
"max_forks_repo_forks_event_min_datetime": "2021-11-04T06:54:45.000Z",
"max_forks_repo_head_hexsha": "7672b7a3185ae77467cc30e05dbe50b36ff2af8a",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "bblfish/agda-categories",
"max_forks_repo_path": "src/Categories/Bicategory/Extras.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "7672b7a3185ae77467cc30e05dbe50b36ff2af8a",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "bblfish/agda-categories",
"max_issues_repo_path": "src/Categories/Bicategory/Extras.agda",
"max_line_length": 122,
"max_stars_count": 5,
"max_stars_repo_head_hexsha": "7672b7a3185ae77467cc30e05dbe50b36ff2af8a",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "bblfish/agda-categories",
"max_stars_repo_path": "src/Categories/Bicategory/Extras.agda",
"max_stars_repo_stars_event_max_datetime": "2020-10-10T21:41:32.000Z",
"max_stars_repo_stars_event_min_datetime": "2020-10-07T12:07:53.000Z",
"num_tokens": 2438,
"size": 4484
} |
open import Relation.Binary.PropositionalEquality using ( refl )
open import Web.Semantic.DL.Category.Object using ( Object )
open import Web.Semantic.DL.Category.Morphism using ( _≣_ )
open import Web.Semantic.DL.Category.Composition using ( _∙_ )
open import Web.Semantic.DL.Category.Tensor using ( _⊗_ ; _⟨⊗⟩_ )
open import Web.Semantic.DL.Category.Unit using ( I )
open import Web.Semantic.DL.Category.Wiring using
( identity ; symm ; assoc ; assoc⁻¹ ; unit₁ ; unit₁⁻¹ ; unit₂ ; unit₂⁻¹ )
open import Web.Semantic.DL.Category.Properties.Wiring using
( rewriting ; rewrite-compose ; rewrite-tensor
; rewrite-identity ; rewrite-symm ; rewrite-assoc ; rewrite-assoc⁻¹
; rewrite-unit₁ ; rewrite-unit₁⁻¹ ; rewrite-unit₂ ; rewrite-unit₂⁻¹ )
open import Web.Semantic.DL.Signature using ( Signature )
open import Web.Semantic.DL.TBox using ( TBox )
open import Web.Semantic.Util using ( _≡⊎≡_ )
module Web.Semantic.DL.Category.Properties.Tensor.Coherence
{Σ : Signature} {S T : TBox Σ} where
assoc-unit : ∀ (A₁ A₂ : Object S T) →
(assoc A₁ I A₂ ∙ (identity A₁ ⟨⊗⟩ unit₁ A₂) ≣ unit₂ A₁ ⟨⊗⟩ identity A₂)
assoc-unit A₁ A₂ = rewriting
(rewrite-compose (rewrite-assoc A₁ I A₂)
(rewrite-tensor (rewrite-identity A₁) (rewrite-unit₁ A₂)))
((λ x → refl) ≡⊎≡ (λ x → refl))
(rewrite-tensor (rewrite-unit₂ A₁) (rewrite-identity A₂))
assoc-assoc : ∀ (A₁ A₂ A₃ A₄ : Object S T) →
(assoc (A₁ ⊗ A₂) A₃ A₄ ∙ assoc A₁ A₂ (A₃ ⊗ A₄) ≣
(assoc A₁ A₂ A₃ ⟨⊗⟩ identity A₄) ∙ assoc A₁ (A₂ ⊗ A₃) A₄ ∙ (identity A₁ ⟨⊗⟩ assoc A₂ A₃ A₄))
assoc-assoc A₁ A₂ A₃ A₄ = rewriting
(rewrite-compose (rewrite-assoc (A₁ ⊗ A₂) A₃ A₄) (rewrite-assoc A₁ A₂ (A₃ ⊗ A₄)))
((λ x → refl) ≡⊎≡ ((λ x → refl) ≡⊎≡ ((λ x → refl) ≡⊎≡ (λ x → refl))))
(rewrite-compose (rewrite-tensor (rewrite-assoc A₁ A₂ A₃) (rewrite-identity A₄))
(rewrite-compose (rewrite-assoc A₁ (A₂ ⊗ A₃) A₄)
(rewrite-tensor (rewrite-identity A₁) (rewrite-assoc A₂ A₃ A₄))))
assoc-symm : ∀ (A₁ A₂ A₃ : Object S T) →
(symm (A₁ ⊗ A₂) A₃ ∙ assoc⁻¹ A₃ A₁ A₂ ≣
assoc A₁ A₂ A₃ ∙ (identity A₁ ⟨⊗⟩ symm A₂ A₃) ∙ assoc⁻¹ A₁ A₃ A₂ ∙ (symm A₁ A₃ ⟨⊗⟩ identity A₂))
assoc-symm A₁ A₂ A₃ = rewriting
(rewrite-compose (rewrite-symm (A₁ ⊗ A₂) A₃) (rewrite-assoc⁻¹ A₃ A₁ A₂))
(((λ x → refl) ≡⊎≡ (λ x → refl)) ≡⊎≡ (λ x → refl))
(rewrite-compose (rewrite-assoc A₁ A₂ A₃)
(rewrite-compose (rewrite-tensor (rewrite-identity A₁) (rewrite-symm A₂ A₃))
(rewrite-compose (rewrite-assoc⁻¹ A₁ A₃ A₂)
(rewrite-tensor (rewrite-symm A₁ A₃) (rewrite-identity A₂)))))
symm-unit : ∀ (A : Object S T) →
(symm A I ∙ unit₁ A ≣ unit₂ A)
symm-unit A = rewriting
(rewrite-compose (rewrite-symm A I) (rewrite-unit₁ A))
(λ x → refl)
(rewrite-unit₂ A)
| {
"alphanum_fraction": 0.6633480826,
"avg_line_length": 49.3090909091,
"ext": "agda",
"hexsha": "94668e32d80340088384e23e1b37057b873c67d8",
"lang": "Agda",
"max_forks_count": 3,
"max_forks_repo_forks_event_max_datetime": "2022-03-12T11:40:03.000Z",
"max_forks_repo_forks_event_min_datetime": "2017-12-03T14:52:09.000Z",
"max_forks_repo_head_hexsha": "38fbc3af7062ba5c3d7d289b2b4bcfb995d99057",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "bblfish/agda-web-semantic",
"max_forks_repo_path": "src/Web/Semantic/DL/Category/Properties/Tensor/Coherence.agda",
"max_issues_count": 4,
"max_issues_repo_head_hexsha": "38fbc3af7062ba5c3d7d289b2b4bcfb995d99057",
"max_issues_repo_issues_event_max_datetime": "2021-01-04T20:57:19.000Z",
"max_issues_repo_issues_event_min_datetime": "2018-11-14T02:32:28.000Z",
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "bblfish/agda-web-semantic",
"max_issues_repo_path": "src/Web/Semantic/DL/Category/Properties/Tensor/Coherence.agda",
"max_line_length": 100,
"max_stars_count": 9,
"max_stars_repo_head_hexsha": "8ddbe83965a616bff6fc7a237191fa261fa78bab",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "agda/agda-web-semantic",
"max_stars_repo_path": "src/Web/Semantic/DL/Category/Properties/Tensor/Coherence.agda",
"max_stars_repo_stars_event_max_datetime": "2020-03-14T14:21:08.000Z",
"max_stars_repo_stars_event_min_datetime": "2015-09-13T17:46:41.000Z",
"num_tokens": 1075,
"size": 2712
} |
module Tactic.Reflection.Substitute where
open import Prelude hiding (abs)
open import Builtin.Reflection
open import Tactic.Reflection.DeBruijn
patternArgsVars : List (Arg Pattern) → Nat
patternVars : Pattern → Nat
patternVars (con _ ps) = patternArgsVars ps
patternVars dot = 1
patternVars (var _) = 1
patternVars (lit x) = 0
patternVars (proj _) = 0
patternVars absurd = 0
patternArgsVars [] = 0
patternArgsVars (arg _ p ∷ ps) = patternVars p + patternArgsVars ps
IsSafe : Term → Set
IsSafe (lam _ _) = ⊥
IsSafe _ = ⊤
data SafeTerm : Set where
safe : (v : Term) (p : IsSafe v) → SafeTerm
maybeSafe : Term → Maybe SafeTerm
maybeSafe (var x args) = just (safe (var x args) _)
maybeSafe (con c args) = just (safe (con c args) _)
maybeSafe (def f args) = just (safe (def f args) _)
maybeSafe (meta x args) = just (safe (meta x args) _)
maybeSafe (lam v t) = nothing
maybeSafe (pat-lam cs args) = just (safe (pat-lam cs args) _)
maybeSafe (pi a b) = just (safe (pi a b) _)
maybeSafe (agda-sort s) = just (safe (agda-sort s) _)
maybeSafe (lit l) = just (safe (lit l) _)
maybeSafe unknown = just (safe unknown _)
instance
DeBruijnSafeTerm : DeBruijn SafeTerm
strengthenFrom {{DeBruijnSafeTerm}} k n (safe v _) = do
-- Strengthening or weakening safe terms always results in safe terms,
-- but proving that is a bit of a bother, thus maybeSafe.
v₁ ← strengthenFrom k n v
maybeSafe v₁
weakenFrom {{DeBruijnSafeTerm}} k n (safe v p) =
maybe (safe unknown _) id (maybeSafe (weakenFrom k n v))
safe-term : SafeTerm → Term
safe-term (safe v _) = v
applyTerm : SafeTerm → List (Arg Term) → Term
applyTerm v [] = safe-term v
applyTerm (safe (var x args) _) args₁ = var x (args ++ args₁)
applyTerm (safe (con c args) _) args₁ = con c (args ++ args₁)
applyTerm (safe (def f args) _) args₁ = def f (args ++ args₁)
applyTerm (safe (meta x args) _) args₁ = meta x (args ++ args₁)
applyTerm (safe (lam v t) ()) args
applyTerm (safe (pat-lam cs args) _) args₁ = pat-lam cs (args ++ args₁)
applyTerm (safe (pi a b) _) _ = pi a b
applyTerm (safe (agda-sort s) _) _ = agda-sort s
applyTerm (safe (lit l) _) _ = lit l
applyTerm (safe unknown _) _ = unknown
Subst : Set → Set
Subst A = List SafeTerm → A → A
substTerm : Subst Term
substArgs : Subst (List (Arg Term))
substArg : Subst (Arg Term)
substAbs : Subst (Abs Term)
substSort : Subst Sort
substClauses : Subst (List Clause)
substClause : Subst Clause
substTerm σ (var x args) =
case index σ x of λ
{ nothing → var (x - length σ) (substArgs σ args)
; (just v) → applyTerm v (substArgs σ args) }
substTerm σ (con c args) = con c (substArgs σ args)
substTerm σ (def f args) = def f (substArgs σ args)
substTerm σ (meta x args) = meta x (substArgs σ args)
substTerm σ (lam v b) = lam v (substAbs σ b)
substTerm σ (pat-lam cs args) = pat-lam (substClauses σ cs) (substArgs σ args)
substTerm σ (pi a b) = pi (substArg σ a) (substAbs σ b)
substTerm σ (agda-sort s) = agda-sort (substSort σ s)
substTerm σ (lit l) = lit l
substTerm σ unknown = unknown
substSort σ (set t) = set (substTerm σ t)
substSort σ (lit n) = lit n
substSort σ unknown = unknown
substClauses σ [] = []
substClauses σ (c ∷ cs) = substClause σ c ∷ substClauses σ cs
substClause σ (clause ps b) =
case patternArgsVars ps of λ
{ zero → clause ps (substTerm σ b)
; (suc n) → clause ps (substTerm (reverse (map (λ i → safe (var i []) _) (from 0 to n)) ++ weaken (suc n) σ) b)
}
substClause σ (absurd-clause ps) = absurd-clause ps
substArgs σ [] = []
substArgs σ (x ∷ args) = substArg σ x ∷ substArgs σ args
substArg σ (arg i x) = arg i (substTerm σ x)
substAbs σ (abs x v) = abs x $ substTerm (safe (var 0 []) _ ∷ weaken 1 σ) v
private
toArgs : Nat → List (Arg SafeTerm) → List (Arg Term)
toArgs k = map (λ x → weaken k (fmap safe-term x))
SafeApplyType : Set → Set
SafeApplyType A = List SafeTerm → Nat → A → List (Arg SafeTerm) → A
safeApplyAbs : SafeApplyType (Abs Term)
safeApplyArg : SafeApplyType (Arg Term)
safeApplySort : SafeApplyType Sort
-- safeApply′ env |Θ| v args = v′
-- where Γ, Δ, Θ ⊢ v
-- Γ ⊢ env : Δ
-- Γ ⊢ args
-- Γ, Θ ⊢ v′
safeApply′ : List SafeTerm → Nat → Term → List (Arg SafeTerm) → Term
safeApply′ env k (var x args) args₁ =
if x <? k then var x (args ++ toArgs k args₁)
else case index env (x - k) of λ
{ nothing → var (x - length env) (args ++ toArgs k args₁)
; (just v) → applyTerm v (args ++ toArgs k args₁) }
safeApply′ env k (con c args) args₁ = con c (args ++ toArgs k args₁)
safeApply′ env k (def f args) args₁ = def f (args ++ toArgs k args₁)
safeApply′ env k (lam v t) (a ∷ args₁) = safeApply′ (unArg a ∷ env) k (unAbs t) args₁
safeApply′ env k (lam v b) [] = lam v $ safeApplyAbs env k b []
safeApply′ env k (pat-lam cs args) args₁ = pat-lam cs (args ++ toArgs k args₁)
-- not right if applying to constructors
safeApply′ env k (pi a b) _ = pi (safeApplyArg env k a []) (safeApplyAbs env k b [])
safeApply′ env k (agda-sort s) args₁ = agda-sort (safeApplySort env k s [])
safeApply′ env k (lit l) args₁ = lit l
safeApply′ env k (meta x args) args₁ = meta x (args ++ toArgs k args₁)
safeApply′ env k unknown args₁ = unknown
safeApplyAbs env k (abs x b) _ = abs x (safeApply′ env (suc k) b [])
safeApplyArg env k (arg i v) args₁ = arg i (safeApply′ env k v args₁)
safeApplySort env k (set t) _ = set (safeApply′ env k t [])
safeApplySort env k (lit n) _ = lit n
safeApplySort env k unknown _ = unknown
safeApply : Term → List (Arg SafeTerm) → Term
safeApply v args = safeApply′ [] 0 v args
| {
"alphanum_fraction": 0.6379012772,
"avg_line_length": 37.8692810458,
"ext": "agda",
"hexsha": "8616c233651a6e15b040e40d2a401ad5df4fe211",
"lang": "Agda",
"max_forks_count": null,
"max_forks_repo_forks_event_max_datetime": null,
"max_forks_repo_forks_event_min_datetime": null,
"max_forks_repo_head_hexsha": "75016b4151ed601e28f4462cd7b6b1aaf5d0d1a6",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "lclem/agda-prelude",
"max_forks_repo_path": "src/Tactic/Reflection/Substitute.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "75016b4151ed601e28f4462cd7b6b1aaf5d0d1a6",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "lclem/agda-prelude",
"max_issues_repo_path": "src/Tactic/Reflection/Substitute.agda",
"max_line_length": 113,
"max_stars_count": null,
"max_stars_repo_head_hexsha": "75016b4151ed601e28f4462cd7b6b1aaf5d0d1a6",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "lclem/agda-prelude",
"max_stars_repo_path": "src/Tactic/Reflection/Substitute.agda",
"max_stars_repo_stars_event_max_datetime": null,
"max_stars_repo_stars_event_min_datetime": null,
"num_tokens": 1897,
"size": 5794
} |
module _ where
{-# BUILTIN INTERVAL I #-}
| {
"alphanum_fraction": 0.6511627907,
"avg_line_length": 10.75,
"ext": "agda",
"hexsha": "72e65171c96d464e4972b1d0a1610811bb04aa77",
"lang": "Agda",
"max_forks_count": 371,
"max_forks_repo_forks_event_max_datetime": "2022-03-30T19:00:30.000Z",
"max_forks_repo_forks_event_min_datetime": "2015-01-03T14:04:08.000Z",
"max_forks_repo_head_hexsha": "7f58030124fa99dfbf8db376659416f3ad8384de",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "cruhland/agda",
"max_forks_repo_path": "test/Fail/Issue2788a.agda",
"max_issues_count": 4066,
"max_issues_repo_head_hexsha": "7f58030124fa99dfbf8db376659416f3ad8384de",
"max_issues_repo_issues_event_max_datetime": "2022-03-31T21:14:49.000Z",
"max_issues_repo_issues_event_min_datetime": "2015-01-10T11:24:51.000Z",
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "cruhland/agda",
"max_issues_repo_path": "test/Fail/Issue2788a.agda",
"max_line_length": 26,
"max_stars_count": 1989,
"max_stars_repo_head_hexsha": "7f58030124fa99dfbf8db376659416f3ad8384de",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "cruhland/agda",
"max_stars_repo_path": "test/Fail/Issue2788a.agda",
"max_stars_repo_stars_event_max_datetime": "2022-03-30T18:20:48.000Z",
"max_stars_repo_stars_event_min_datetime": "2015-01-09T23:51:16.000Z",
"num_tokens": 10,
"size": 43
} |
import Oscar.Class.Reflexivity.Function
import Oscar.Class.Transextensionality.Proposequality -- FIXME why not use the instance here?
open import Oscar.Class
open import Oscar.Class.Category
open import Oscar.Class.HasEquivalence
open import Oscar.Class.IsCategory
open import Oscar.Class.IsPrecategory
open import Oscar.Class.Precategory
open import Oscar.Class.Reflexivity
open import Oscar.Class.Transassociativity
open import Oscar.Class.Transextensionality
open import Oscar.Class.Transitivity
open import Oscar.Class.Transleftidentity
open import Oscar.Class.Transrightidentity
open import Oscar.Class.[IsExtensionB]
open import Oscar.Data.Proposequality
open import Oscar.Prelude
open import Oscar.Property.Category.Function
open import Oscar.Property.Setoid.Proposextensequality
module Oscar.Property.Category.ExtensionProposextensequality where
module _
{a} {A : Ø a} {b} {B : A → Ø b}
where
instance
𝓣ransassociativityExtensionProposextensequality : Transassociativity.class (Extension B) Proposextensequality transitivity
𝓣ransassociativityExtensionProposextensequality .⋆ _ _ _ _ = !
module _
{a} {A : Ø a} {b} {B : A → Ø b}
where
instance
𝓣ransextensionalityExtensionProposextensequality : Transextensionality.class (Extension B) Proposextensequality transitivity
𝓣ransextensionalityExtensionProposextensequality .⋆ = 𝓣ransextensionalityFunctionProposextensequality .⋆
-- 𝓣ransextensionalityExtensionProposextensequality .⋆ {f₂ = f₂} f₁≡̇f₂ g₁≡̇g₂ x rewrite f₁≡̇f₂ x = g₁≡̇g₂ (f₂ x) -- FIXME using this causes problems in Test.Functor
module _
{a} {A : Ø a} {b} {B : A → Ø b}
where
instance
𝓣ransleftidentityExtensionProposextensequality : Transleftidentity.class (Extension B) Proposextensequality ε transitivity
𝓣ransleftidentityExtensionProposextensequality .⋆ _ = !
module _
{a} {A : Ø a} {b} {B : A → Ø b}
where
instance
𝓣ransrightidentityExtensionProposextensequality : Transrightidentity.class (Extension B) Proposextensequality ε transitivity
𝓣ransrightidentityExtensionProposextensequality .⋆ _ = !
module _
{a} {A : Ø a} {b} {B : A → Ø b}
where
instance
HasEquivalenceExtension : ∀ {x y : A} ⦃ _ : [IsExtensionB] B ⦄ → HasEquivalence (Extension B x y) _
HasEquivalenceExtension = ∁ Proposextensequality
module _
{a} {A : Ø a} {b} {B : A → Ø b}
where
instance
IsPrecategoryExtension : IsPrecategory (Extension B) Proposextensequality transitivity
IsPrecategoryExtension = ∁
IsCategoryExtension : IsCategory (Extension B) Proposextensequality ε transitivity
IsCategoryExtension = ∁
module _
{a} {A : Ø a} {b} (B : A → Ø b)
where
PrecategoryExtension : Precategory _ _ _
PrecategoryExtension = ∁ (Extension B) Proposextensequality transitivity
CategoryExtension : Category _ _ _
CategoryExtension = ∁ (Extension B) Proposextensequality ε transitivity
| {
"alphanum_fraction": 0.768515329,
"avg_line_length": 31.9010989011,
"ext": "agda",
"hexsha": "407cf230274dd9e067bdcb0c7382cdcd559ea098",
"lang": "Agda",
"max_forks_count": null,
"max_forks_repo_forks_event_max_datetime": null,
"max_forks_repo_forks_event_min_datetime": null,
"max_forks_repo_head_hexsha": "52e1cdbdee54d9a8eaee04ee518a0d7f61d25afb",
"max_forks_repo_licenses": [
"RSA-MD"
],
"max_forks_repo_name": "m0davis/oscar",
"max_forks_repo_path": "archive/agda-3/src/Oscar/Property/Category/ExtensionProposextensequality.agda",
"max_issues_count": 1,
"max_issues_repo_head_hexsha": "52e1cdbdee54d9a8eaee04ee518a0d7f61d25afb",
"max_issues_repo_issues_event_max_datetime": "2019-05-11T23:33:04.000Z",
"max_issues_repo_issues_event_min_datetime": "2019-04-29T00:35:04.000Z",
"max_issues_repo_licenses": [
"RSA-MD"
],
"max_issues_repo_name": "m0davis/oscar",
"max_issues_repo_path": "archive/agda-3/src/Oscar/Property/Category/ExtensionProposextensequality.agda",
"max_line_length": 169,
"max_stars_count": null,
"max_stars_repo_head_hexsha": "52e1cdbdee54d9a8eaee04ee518a0d7f61d25afb",
"max_stars_repo_licenses": [
"RSA-MD"
],
"max_stars_repo_name": "m0davis/oscar",
"max_stars_repo_path": "archive/agda-3/src/Oscar/Property/Category/ExtensionProposextensequality.agda",
"max_stars_repo_stars_event_max_datetime": null,
"max_stars_repo_stars_event_min_datetime": null,
"num_tokens": 850,
"size": 2903
} |
{-# OPTIONS --without-K #-}
open import lib.Basics
open import lib.NType2
open import lib.Equivalences2
open import lib.NConnected
open import lib.types.Nat
open import lib.types.Pi
open import lib.types.Sigma
open import lib.types.TLevel
open import lib.types.Truncation
open import lib.types.Group
open import lib.types.Pointed
open import lib.types.LoopSpace
open import lib.groups.Homomorphisms
open import lib.groups.HomotopyGroup
module lib.types.EilenbergMacLane1 where
module EM₁ {i} (G : Group i) where
module G = Group G
private
data #EM₁-aux : Type i where
#embase : #EM₁-aux
data #EM₁ : Type i where
#em₁ : #EM₁-aux → (Unit → Unit) → #EM₁
EM₁ : Type i
EM₁ = #EM₁
embase : EM₁
embase = #em₁ #embase _
⊙EM₁ : Ptd i
⊙EM₁ = ⊙[ EM₁ , embase ]
postulate -- HIT
emlevel : has-level ⟨ 1 ⟩ EM₁
emloop : G.El → embase == embase
emloop-ident : emloop G.ident == idp
emloop-comp : ∀ g₁ g₂ → emloop (G.comp g₁ g₂) == emloop g₁ ∙ emloop g₂
module EM₁Rec {j} {C : Type j}
(C-level : has-level ⟨ 1 ⟩ C)
(embase* : C)
(hom* : G →ᴳ (Ω^S-group 0 (C , embase*) C-level)) where
f : EM₁ → C
f (#em₁ #embase _) = embase*
postulate -- HIT
emloop-β : (g : G.El) → ap f (emloop g) == GroupHom.f hom* g
open EM₁Rec public using () renaming (f to EM₁-rec)
module EM₁Elim {j} {P : EM₁ → Type j}
(P-level : (x : EM₁) → has-level ⟨ 1 ⟩ (P x))
(embase* : P embase)
(emloop* : (g : G.El) → embase* == embase* [ P ↓ emloop g ])
(preserves-ident : emloop* G.ident == idp
[ (λ p → embase* == embase* [ P ↓ p ]) ↓ emloop-ident ])
(preserves-comp : (g₁ g₂ : G.El) →
emloop* (G.comp g₁ g₂) == emloop* g₁ ∙ᵈ emloop* g₂
[ (λ p → embase* == embase* [ P ↓ p ]) ↓ emloop-comp g₁ g₂ ])
where
f : Π EM₁ P
f (#em₁ #embase _) = embase*
postulate -- HIT
emloop-β : (g : G.El) → apd f (emloop g) == emloop* g
open EM₁Elim public using () renaming (f to EM₁-elim)
emloop-inv : ∀ g → emloop (G.inv g) == ! (emloop g)
emloop-inv g = cancels-inverse _ _ lemma
where
cancels-inverse : ∀ {i} {A : Type i} {x y : A}
(p : x == y) (q : y == x) → p ∙ q == idp → p == ! q
cancels-inverse p idp r = ! (∙-unit-r p) ∙ r
lemma : emloop (G.inv g) ∙ emloop g == idp
lemma = ! (emloop-comp (G.inv g) g) ∙ ap emloop (G.invl g) ∙ emloop-ident
module π₁ where
comp-equiv : ∀ g → G.El ≃ G.El
comp-equiv g = equiv
(λ x → G.comp x g)
(λ x → G.comp x (G.inv g))
(λ x → G.assoc x (G.inv g) g ∙ ap (G.comp x) (G.invl g) ∙ G.unitr x)
(λ x → G.assoc x g (G.inv g) ∙ ap (G.comp x) (G.invr g) ∙ G.unitr x)
comp-equiv-id : comp-equiv G.ident == ide G.El
comp-equiv-id =
pair= (λ= G.unitr)
(prop-has-all-paths-↓ {B = is-equiv} (is-equiv-is-prop $ idf G.El))
comp-equiv-comp : (g₁ g₂ : G.El) → comp-equiv (G.comp g₁ g₂)
== (comp-equiv g₂ ∘e comp-equiv g₁)
comp-equiv-comp g₁ g₂ =
pair= (λ= (λ x → ! (G.assoc x g₁ g₂)))
(prop-has-all-paths-↓ {B = is-equiv} (is-equiv-is-prop _))
Ω-group : Group (lsucc i)
Ω-group = group (G.El == G.El) (universe-=-level G.El-level G.El-level)
(Ω^S-group-structure 0 (Type i , G.El))
0-group : Group (lsucc i)
0-group = Ω^S-group 0
((0 -Type i) , (G.El , G.El-level)) (0 -Type-level i)
Codes-hom₁ : G →ᴳ Ω-group
Codes-hom₁ = record {
f = ua ∘ comp-equiv;
pres-comp = λ g₁ g₂ →
ua (comp-equiv (G.comp g₁ g₂))
=⟨ ap ua (comp-equiv-comp g₁ g₂) ⟩
ua (comp-equiv g₂ ∘e comp-equiv g₁)
=⟨ ua-∘e (comp-equiv g₁) (comp-equiv g₂) ⟩
ua (comp-equiv g₁) ∙ ua (comp-equiv g₂) ∎}
Codes-hom₂ : Ω-group →ᴳ 0-group
Codes-hom₂ = record {
f = λ p → pair= p (phap p);
pres-comp = λ p₁ p₂ →
pair= (p₁ ∙ p₂) (phap (p₁ ∙ p₂))
=⟨ prop-has-all-paths (↓-level (λ _ →
raise-level _ has-level-is-prop)) _ _
|in-ctx (λ w → pair= (p₁ ∙ p₂) w) ⟩
pair= (p₁ ∙ p₂) (phap p₁ ∙ᵈ phap p₂)
=⟨ ! (Σ-∙ (phap p₁) (phap p₂)) ⟩
pair= p₁ (phap p₁) ∙ pair= p₂ (phap p₂) ∎}
where
-- saving some space
phap : (p : G.El == G.El)
→ G.El-level == G.El-level [ has-level 0 ↓ p ]
phap p = prop-has-all-paths-↓ has-level-is-prop
Codes-hom : G →ᴳ 0-group
Codes-hom = Codes-hom₂ ∘ᴳ Codes-hom₁
Codes : EM₁ → 0 -Type i
Codes = EM₁-rec {C = 0 -Type i} (0 -Type-level i)
(G.El , G.El-level)
Codes-hom
abstract
↓-Codes-loop : ∀ g g' → g' == G.comp g' g [ fst ∘ Codes ↓ emloop g ]
↓-Codes-loop g g' =
↓-ap-out fst Codes (emloop g) $
↓-ap-out (idf _) fst (ap Codes (emloop g)) $
transport (λ w → g' == G.comp g' g [ idf _ ↓ ap fst w ])
(! (EM₁Rec.emloop-β (0 -Type-level i)
(G.El , G.El-level) Codes-hom g)) $
transport (λ w → g' == G.comp g' g [ idf _ ↓ w ])
(! (fst=-β (ua $ comp-equiv g) _)) $
↓-idf-ua-in (comp-equiv g) idp
encode : {x : EM₁} → embase == x → fst (Codes x)
encode α = transport (fst ∘ Codes) α G.ident
encode-emloop : ∀ g → encode (emloop g) == g
encode-emloop g = to-transp $
transport (λ x → G.ident == x [ fst ∘ Codes ↓ emloop g ])
(G.unitl g) (↓-Codes-loop g G.ident)
decode : {x : EM₁} → fst (Codes x) → embase == x
decode {x} =
EM₁-elim {P = λ x' → fst (Codes x') → embase == x'}
(λ _ → Π-level (λ _ → =-preserves-level _ emlevel))
emloop
loop'
(prop-has-all-paths-↓ (Π-level (λ _ → emlevel _ _) _ _))
(λ _ _ → prop-has-all-paths-↓ (↓-level (λ _ → Π-level (λ _ → emlevel _ _))))
x
where
loop' : (g : G.El)
→ emloop == emloop [ (λ x' → fst (Codes x') → embase == x') ↓ emloop g ]
loop' g = ↓-→-from-transp $ λ= $ λ y →
transport (λ z → embase == z) (emloop g) (emloop y)
=⟨ trans-pathfrom (emloop g) (emloop y) ⟩
emloop y ∙ emloop g
=⟨ ! (emloop-comp y g) ⟩
emloop (G.comp y g)
=⟨ ap emloop (! (to-transp (↓-Codes-loop g y))) ⟩
emloop (transport (λ z → fst (Codes z)) (emloop g) y) ∎
decode-encode : ∀ {x} (α : embase == x) → decode (encode α) == α
decode-encode idp = emloop-ident
abstract
Ω¹-equiv : (embase == embase) ≃ G.El
Ω¹-equiv = equiv encode emloop encode-emloop decode-encode
abstract
Ω¹-path : (embase == embase) == G.El
Ω¹-path = ua Ω¹-equiv
abstract
π₁-path : Trunc 0 (embase == embase) == G.El
π₁-path = ap (Trunc 0) Ω¹-path ∙ ua (unTrunc-equiv G.El G.El-level)
abstract
π₁-iso : πS 0 (EM₁ , embase) == G
π₁-iso = ! $ group-ua
(record { f = [_] ∘ emloop;
pres-comp = λ g₁ g₂ → ap [_] (emloop-comp g₁ g₂) } ,
snd ((unTrunc-equiv (embase == embase) (emlevel _ _))⁻¹
∘e (Ω¹-equiv ⁻¹)))
{- EM₁ is 0-connected -}
abstract
EM₁-conn : is-connected 0 EM₁
EM₁-conn = ([ embase ] , Trunc-elim (λ _ → =-preserves-level _ Trunc-level)
(EM₁-elim
{P = λ x → [ embase ] == [ x ]}
(λ _ → raise-level _ (=-preserves-level _ Trunc-level))
idp
(λ _ → prop-has-all-paths-↓ (Trunc-level {n = 0} _ _))
(set-↓-has-all-paths-↓ (=-preserves-level _ Trunc-level))
(λ _ _ → set-↓-has-all-paths-↓ (=-preserves-level _ Trunc-level))))
| {
"alphanum_fraction": 0.5175496253,
"avg_line_length": 33.0739130435,
"ext": "agda",
"hexsha": "7f327f4b57d76749307e6ae3815fe06bc75ba0b2",
"lang": "Agda",
"max_forks_count": null,
"max_forks_repo_forks_event_max_datetime": null,
"max_forks_repo_forks_event_min_datetime": null,
"max_forks_repo_head_hexsha": "bc849346a17b33e2679a5b3f2b8efbe7835dc4b6",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "cmknapp/HoTT-Agda",
"max_forks_repo_path": "core/lib/types/EilenbergMacLane1.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "bc849346a17b33e2679a5b3f2b8efbe7835dc4b6",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "cmknapp/HoTT-Agda",
"max_issues_repo_path": "core/lib/types/EilenbergMacLane1.agda",
"max_line_length": 84,
"max_stars_count": null,
"max_stars_repo_head_hexsha": "bc849346a17b33e2679a5b3f2b8efbe7835dc4b6",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "cmknapp/HoTT-Agda",
"max_stars_repo_path": "core/lib/types/EilenbergMacLane1.agda",
"max_stars_repo_stars_event_max_datetime": null,
"max_stars_repo_stars_event_min_datetime": null,
"num_tokens": 2790,
"size": 7607
} |
module Issue1362 where
open import Common.Prelude
open import Common.Equality
open import Common.Reflection
module M₁ (A₁ : Set) where
data D (B : Set) : Set where
type₁ : TC Type
type₁ = getType (quote D)
module M₂ (A₂ : Set) where
open M₁ A₂
type₂ : TC Type
type₂ = getType (quote D)
open M₁ Nat
open M₂ Nat
foo : type₁ ≡ type₂
foo = cong getType {quote D} {quote D} ?
| {
"alphanum_fraction": 0.6862244898,
"avg_line_length": 15.0769230769,
"ext": "agda",
"hexsha": "b7a5cd7434b0a3bf42343cda1de56ac40820c9cd",
"lang": "Agda",
"max_forks_count": 371,
"max_forks_repo_forks_event_max_datetime": "2022-03-30T19:00:30.000Z",
"max_forks_repo_forks_event_min_datetime": "2015-01-03T14:04:08.000Z",
"max_forks_repo_head_hexsha": "231d6ad8e77b67ff8c4b1cb35a6c31ccd988c3e9",
"max_forks_repo_licenses": [
"BSD-3-Clause"
],
"max_forks_repo_name": "Agda-zh/agda",
"max_forks_repo_path": "test/Fail/Issue1362.agda",
"max_issues_count": 4066,
"max_issues_repo_head_hexsha": "ed8ac6f4062ea8a20fa0f62d5db82d4e68278338",
"max_issues_repo_issues_event_max_datetime": "2022-03-31T21:14:49.000Z",
"max_issues_repo_issues_event_min_datetime": "2015-01-10T11:24:51.000Z",
"max_issues_repo_licenses": [
"BSD-3-Clause"
],
"max_issues_repo_name": "shlevy/agda",
"max_issues_repo_path": "test/Fail/Issue1362.agda",
"max_line_length": 40,
"max_stars_count": 1989,
"max_stars_repo_head_hexsha": "ed8ac6f4062ea8a20fa0f62d5db82d4e68278338",
"max_stars_repo_licenses": [
"BSD-3-Clause"
],
"max_stars_repo_name": "shlevy/agda",
"max_stars_repo_path": "test/Fail/Issue1362.agda",
"max_stars_repo_stars_event_max_datetime": "2022-03-30T18:20:48.000Z",
"max_stars_repo_stars_event_min_datetime": "2015-01-09T23:51:16.000Z",
"num_tokens": 128,
"size": 392
} |
{-# OPTIONS --without-K #-}
open import HoTT
open import cohomology.Exactness
open import cohomology.FunctionOver
module cohomology.ProductRepr where
{- Given the following commutative diagram of homomorphisms,
H₁ i₁ i₂ H₂
↘ ↙
id ↓ G ↓ id
↙ ↘
H₁ j₁ j₂ H₂
- there exists an isomorphism G == H₁ × H₂ such that i₁,i₂ correspond
- to the natural injections and j₁,j₂ correspond to the natural
- projections. -}
module ProductRepr {i j}
{G : Group (lmax i j)} {H₁ : Group i} {H₂ : Group j}
(i₁ : H₁ →ᴳ G) (i₂ : H₂ →ᴳ G) (j₁ : G →ᴳ H₁) (j₂ : G →ᴳ H₂)
(p₁ : ∀ h₁ → GroupHom.f j₁ (GroupHom.f i₁ h₁) == h₁)
(p₂ : ∀ h₂ → GroupHom.f j₂ (GroupHom.f i₂ h₂) == h₂)
(ex₁ : is-exact (GroupHom.⊙f i₁) (GroupHom.⊙f j₂))
(ex₂ : is-exact (GroupHom.⊙f i₂) (GroupHom.⊙f j₁))
where
zero-ker : (g : Group.El G)
→ GroupHom.f (×ᴳ-hom-in j₁ j₂) g == Group.ident (H₁ ×ᴳ H₂)
→ g == Group.ident G
zero-ker g q = Trunc-rec (Group.El-level G _ _)
(lemma g (fst×= q))
(ktoi ex₁ g (snd×= q))
where
lemma : (g : Group.El G) (r : GroupHom.f j₁ g == Group.ident H₁)
→ Σ (Group.El H₁) (λ h → GroupHom.f i₁ h == g)
→ g == Group.ident G
lemma ._ r (h , idp) =
ap (GroupHom.f i₁) (! (p₁ h) ∙ r) ∙ GroupHom.pres-ident i₁
β₁ : (h₁ : Group.El H₁) (h₂ : Group.El H₂)
→ GroupHom.f j₁ (Group.comp G (GroupHom.f i₁ h₁) (GroupHom.f i₂ h₂)) == h₁
β₁ h₁ h₂ =
GroupHom.pres-comp j₁ (GroupHom.f i₁ h₁) (GroupHom.f i₂ h₂)
∙ ap2 (Group.comp H₁) (p₁ h₁) (itok ex₂ _ [ h₂ , idp ])
∙ Group.unitr H₁ h₁
β₂ : (h₁ : Group.El H₁) (h₂ : Group.El H₂)
→ GroupHom.f j₂ (Group.comp G (GroupHom.f i₁ h₁) (GroupHom.f i₂ h₂)) == h₂
β₂ h₁ h₂ =
GroupHom.pres-comp j₂ (GroupHom.f i₁ h₁) (GroupHom.f i₂ h₂)
∙ ap2 (Group.comp H₂) (itok ex₁ _ [ h₁ , idp ]) (p₂ h₂)
∙ Group.unitl H₂ h₂
iso : G == H₁ ×ᴳ H₂
iso = surj-inj-= (×ᴳ-hom-in j₁ j₂)
(zero-kernel-injective (×ᴳ-hom-in j₁ j₂) zero-ker)
(λ {(h₁ , h₂) → [ Group.comp G (GroupHom.f i₁ h₁) (GroupHom.f i₂ h₂) ,
pair×= (β₁ h₁ h₂) (β₂ h₁ h₂) ]})
fst-over : j₁ == ×ᴳ-fst [ (λ U → U →ᴳ H₁) ↓ iso ]
fst-over = domain-over-iso _ _ _ _ $ domain-over-equiv fst _
snd-over : j₂ == ×ᴳ-snd {G = H₁} [ (λ U → U →ᴳ H₂) ↓ iso ]
snd-over = domain-over-iso _ _ _ _ $ domain-over-equiv snd _
inl-over : i₁ == ×ᴳ-inl [ (λ V → H₁ →ᴳ V) ↓ iso ]
inl-over = codomain-over-iso _ _ _ _ $
codomain-over-equiv (GroupHom.f i₁) _
▹ λ= (λ h₁ → pair×= (p₁ h₁) (itok ex₁ _ [ h₁ , idp ]))
inr-over : i₂ == ×ᴳ-inr {G = H₁} [ (λ V → H₂ →ᴳ V) ↓ iso ]
inr-over = codomain-over-iso _ _ _ _ $
codomain-over-equiv (GroupHom.f i₂) _
▹ λ= (λ h₂ → pair×= (itok ex₂ _ [ h₂ , idp ]) (p₂ h₂))
{- Given additionally maps
i₀ j₀
K –––→ G ––→ L
- such that j₀∘i₀ = 0, we have j₀(i₁(j₁(i₀ k)))⁻¹ = j₀(i₂(j₂(i₀ k))).
- (This is called the hexagon lemma in Eilenberg & Steenrod's book.
- The hexagon is not visible in this presentation.)
-}
module HexagonLemma {k l}
{K : Group k} {L : Group l}
(i₀ : K →ᴳ G) (j₀ : G →ᴳ L)
(ex₀ : ∀ g → GroupHom.f j₀ (GroupHom.f i₀ g) == Group.ident L)
where
decomp : ∀ g → Group.comp G (GroupHom.f i₁ (GroupHom.f j₁ g))
(GroupHom.f i₂ (GroupHom.f j₂ g))
== g
decomp = transport
(λ {(G' , i₁' , i₂' , j₁' , j₂') → ∀ g →
Group.comp G' (GroupHom.f i₁' (GroupHom.f j₁' g))
(GroupHom.f i₂' (GroupHom.f j₂' g))
== g})
(! (pair= iso (↓-×-in inl-over (↓-×-in inr-over
(↓-×-in fst-over snd-over)))))
(λ {(h₁ , h₂) → pair×= (Group.unitr H₁ h₁) (Group.unitl H₂ h₂)})
cancel : ∀ k →
Group.comp L (GroupHom.f (j₀ ∘ᴳ i₁ ∘ᴳ j₁ ∘ᴳ i₀) k)
(GroupHom.f (j₀ ∘ᴳ i₂ ∘ᴳ j₂ ∘ᴳ i₀) k)
== Group.ident L
cancel k = ! (GroupHom.pres-comp j₀ _ _)
∙ ap (GroupHom.f j₀) (decomp (GroupHom.f i₀ k))
∙ ex₀ k
inv₁ : ∀ k → Group.inv L (GroupHom.f (j₀ ∘ᴳ i₁ ∘ᴳ j₁ ∘ᴳ i₀) k)
== GroupHom.f (j₀ ∘ᴳ i₂ ∘ᴳ j₂ ∘ᴳ i₀) k
inv₁ k = group-inv-unique-r L _ _ (cancel k)
inv₂ : ∀ k → Group.inv L (GroupHom.f (j₀ ∘ᴳ i₂ ∘ᴳ j₂ ∘ᴳ i₀) k)
== GroupHom.f (j₀ ∘ᴳ i₁ ∘ᴳ j₁ ∘ᴳ i₀) k
inv₂ k = group-inv-unique-l L _ _ (cancel k)
| {
"alphanum_fraction": 0.5262919311,
"avg_line_length": 35.8699186992,
"ext": "agda",
"hexsha": "197cf60640f11c3f68b2886efe402b5af1f6bfd1",
"lang": "Agda",
"max_forks_count": null,
"max_forks_repo_forks_event_max_datetime": null,
"max_forks_repo_forks_event_min_datetime": null,
"max_forks_repo_head_hexsha": "1695a7f3dc60177457855ae846bbd86fcd96983e",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "danbornside/HoTT-Agda",
"max_forks_repo_path": "cohomology/ProductRepr.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "1695a7f3dc60177457855ae846bbd86fcd96983e",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "danbornside/HoTT-Agda",
"max_issues_repo_path": "cohomology/ProductRepr.agda",
"max_line_length": 78,
"max_stars_count": null,
"max_stars_repo_head_hexsha": "1695a7f3dc60177457855ae846bbd86fcd96983e",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "danbornside/HoTT-Agda",
"max_stars_repo_path": "cohomology/ProductRepr.agda",
"max_stars_repo_stars_event_max_datetime": null,
"max_stars_repo_stars_event_min_datetime": null,
"num_tokens": 1859,
"size": 4412
} |
------------------------------------------------------------------------
-- The Agda standard library
--
-- The unit type and the total relation on unit
------------------------------------------------------------------------
{-# OPTIONS --without-K --safe #-}
open import Agda.Builtin.Equality using (_≡_)
module Data.Unit.Base where
------------------------------------------------------------------------
-- A unit type defined as a record type
-- Note that by default the unit type is not universe polymorphic as it
-- often results in unsolved metas. See `Data.Unit.Polymorphic` for a
-- universe polymorphic variant.
-- Note also that the name of this type is "\top", not T.
open import Agda.Builtin.Unit public
using (⊤; tt)
------------------------------------------------------------------------
-- DEPRECATED NAMES
------------------------------------------------------------------------
-- Please use the new names as continuing support for the old names is
-- not guaranteed.
-- Version 1.2
record _≤_ (x y : ⊤) : Set where
{-# WARNING_ON_USAGE _≤_
"Warning: _≤_ was deprecated in v1.2.
Please use _≡_ from Relation.Binary.PropositionalEquality instead."
#-}
| {
"alphanum_fraction": 0.4970414201,
"avg_line_length": 31.1315789474,
"ext": "agda",
"hexsha": "e045135e5688f8cea587a1d9294e7c23f3a1849b",
"lang": "Agda",
"max_forks_count": 1,
"max_forks_repo_forks_event_max_datetime": "2021-11-04T06:54:45.000Z",
"max_forks_repo_forks_event_min_datetime": "2021-11-04T06:54:45.000Z",
"max_forks_repo_head_hexsha": "fb380f2e67dcb4a94f353dbaec91624fcb5b8933",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "DreamLinuxer/popl21-artifact",
"max_forks_repo_path": "agda-stdlib/src/Data/Unit/Base.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "fb380f2e67dcb4a94f353dbaec91624fcb5b8933",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "DreamLinuxer/popl21-artifact",
"max_issues_repo_path": "agda-stdlib/src/Data/Unit/Base.agda",
"max_line_length": 72,
"max_stars_count": 5,
"max_stars_repo_head_hexsha": "fb380f2e67dcb4a94f353dbaec91624fcb5b8933",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "DreamLinuxer/popl21-artifact",
"max_stars_repo_path": "agda-stdlib/src/Data/Unit/Base.agda",
"max_stars_repo_stars_event_max_datetime": "2020-10-10T21:41:32.000Z",
"max_stars_repo_stars_event_min_datetime": "2020-10-07T12:07:53.000Z",
"num_tokens": 232,
"size": 1183
} |
module _ where
import Imports.Issue1913-M as M
module _ where
import Imports.Issue1913-I as I
accepted₁ : M.D
accepted₁ = I.x
! : ⦃ _ : M.D ⦄ → M.D
! ⦃ x ⦄ = x
accepted₂ : M.D
accepted₂ = !
-- rejected : M.D
-- rejected = I.x
| {
"alphanum_fraction": 0.6041666667,
"avg_line_length": 11.4285714286,
"ext": "agda",
"hexsha": "aee84262281cdfc4606b918a6a24d6bdbc045267",
"lang": "Agda",
"max_forks_count": 371,
"max_forks_repo_forks_event_max_datetime": "2022-03-30T19:00:30.000Z",
"max_forks_repo_forks_event_min_datetime": "2015-01-03T14:04:08.000Z",
"max_forks_repo_head_hexsha": "231d6ad8e77b67ff8c4b1cb35a6c31ccd988c3e9",
"max_forks_repo_licenses": [
"BSD-3-Clause"
],
"max_forks_repo_name": "Agda-zh/agda",
"max_forks_repo_path": "test/Fail/Issue1913b.agda",
"max_issues_count": 4066,
"max_issues_repo_head_hexsha": "ed8ac6f4062ea8a20fa0f62d5db82d4e68278338",
"max_issues_repo_issues_event_max_datetime": "2022-03-31T21:14:49.000Z",
"max_issues_repo_issues_event_min_datetime": "2015-01-10T11:24:51.000Z",
"max_issues_repo_licenses": [
"BSD-3-Clause"
],
"max_issues_repo_name": "shlevy/agda",
"max_issues_repo_path": "test/Fail/Issue1913b.agda",
"max_line_length": 33,
"max_stars_count": 1989,
"max_stars_repo_head_hexsha": "ed8ac6f4062ea8a20fa0f62d5db82d4e68278338",
"max_stars_repo_licenses": [
"BSD-3-Clause"
],
"max_stars_repo_name": "shlevy/agda",
"max_stars_repo_path": "test/Fail/Issue1913b.agda",
"max_stars_repo_stars_event_max_datetime": "2022-03-30T18:20:48.000Z",
"max_stars_repo_stars_event_min_datetime": "2015-01-09T23:51:16.000Z",
"num_tokens": 93,
"size": 240
} |
{-# OPTIONS --without-K #-}
open import Types
open import Functions
open import Paths
open import HLevel
open import Equivalences
module FiberEquivalences {i j k} {A : Set i} {P : A → Set k} {Q : A → Set j}
(f : (x : A) → (P x → Q x)) where
-- We want to prove that if [f] induces an equivalence on the total spaces,
-- then [f] induces an equivalence fiberwise
total-map : Σ A P → Σ A Q
total-map (x , y) = (x , f x y)
module TotalMapEquiv (e : is-equiv total-map) where
total-equiv : Σ A P ≃ Σ A Q
total-equiv = (total-map , e)
-- The inverse is propositionally fiberwise
base-path-inverse : (x : A) (y : Q x) → π₁ ((total-equiv ⁻¹) ☆ (x , y)) ≡ x
base-path-inverse x y = base-path (inverse-right-inverse total-equiv (x , y))
-- And the action of [total-map] on paths is correct on the base path
total-map-fiberwise-on-paths : {u v : Σ A P} (p : u ≡ v)
→ base-path (ap total-map p) ≡ base-path p
total-map-fiberwise-on-paths {u} {.u} refl = refl
-- Here is the fiberwise inverse, we use the inverse of the total map and
-- transform it into a fiberwise map using [base-path-inverse]
inv : ((x : A) → (Q x → P x))
inv x y = transport P (base-path-inverse x y)
(π₂ ((total-equiv ⁻¹) ☆ (x , y)))
-- We prove that [inv] is a right and left inverse to [f]
inv-right-inverse : (x : A) (y : Q x) → f x (inv x y) ≡ y
inv-right-inverse x y =
app-trans _ _ f (base-path (inverse-right-inverse total-equiv (x , y)))
(π₂ (inverse (_ , e) (x , y)))
∘ fiber-path (inverse-right-inverse total-equiv (x , y))
inv-left-inverse : (x : A) (y : P x) → inv x (f x y) ≡ y
inv-left-inverse x y =
ap (λ u → transport P (base-path (inverse-right-inverse total-equiv
(x , f x y))) u)
(lemma2 x y)
∘ (! (trans-concat P (base-path (inverse-right-inverse total-equiv
(x , f x y)))
(! (base-path-inverse x (f x y))) y)
∘ ap (λ p → transport P p y)
(opposite-left-inverse (ap π₁
(inverse-right-inverse total-equiv (x , f x y))))) where
lemma1 : (x : A) (y : P x)
→ base-path-inverse x (f x y)
≡ base-path (inverse-left-inverse total-equiv (x , y))
lemma1 x y = ap base-path (inverse-triangle total-equiv (x , y))
∘ total-map-fiberwise-on-paths _
lemma2 : (x : A) (y : P x)
→ π₂ ((total-equiv ⁻¹) ☆ (x , f x y))
≡ transport P (! (base-path-inverse x (f x y))) y
lemma2 x y = ! (fiber-path (! (inverse-left-inverse total-equiv (x , y))))
∘ ap (λ p → transport P p y)
(ap-opposite π₁ (inverse-left-inverse total-equiv (x , y))
∘ ! (ap ! (lemma1 x y)))
fiberwise-is-equiv : ((x : A) → is-equiv (f x))
fiberwise-is-equiv x = iso-is-eq (f x) (inv x) (inv-right-inverse x)
(inv-left-inverse x)
fiberwise-is-equiv : is-equiv total-map → ((x : A) → is-equiv (f x))
fiberwise-is-equiv = TotalMapEquiv.fiberwise-is-equiv
| {
"alphanum_fraction": 0.5485110471,
"avg_line_length": 40.0384615385,
"ext": "agda",
"hexsha": "a3d0ece8e0790fbba6ef116c62b8ccf66130a18b",
"lang": "Agda",
"max_forks_count": 50,
"max_forks_repo_forks_event_max_datetime": "2022-02-14T03:03:25.000Z",
"max_forks_repo_forks_event_min_datetime": "2015-01-10T01:48:08.000Z",
"max_forks_repo_head_hexsha": "939a2d83e090fcc924f69f7dfa5b65b3b79fe633",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "nicolaikraus/HoTT-Agda",
"max_forks_repo_path": "old/FiberEquivalences.agda",
"max_issues_count": 31,
"max_issues_repo_head_hexsha": "939a2d83e090fcc924f69f7dfa5b65b3b79fe633",
"max_issues_repo_issues_event_max_datetime": "2021-10-03T19:15:25.000Z",
"max_issues_repo_issues_event_min_datetime": "2015-03-05T20:09:00.000Z",
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "nicolaikraus/HoTT-Agda",
"max_issues_repo_path": "old/FiberEquivalences.agda",
"max_line_length": 79,
"max_stars_count": 294,
"max_stars_repo_head_hexsha": "66f800adef943afdf08c17b8ecfba67340fead5e",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "timjb/HoTT-Agda",
"max_stars_repo_path": "old/FiberEquivalences.agda",
"max_stars_repo_stars_event_max_datetime": "2022-03-20T13:54:45.000Z",
"max_stars_repo_stars_event_min_datetime": "2015-01-09T16:23:23.000Z",
"num_tokens": 940,
"size": 3123
} |
------------------------------------------------------------------------------
-- Agda-Prop Library.
-- Syntax definitions.
------------------------------------------------------------------------------
open import Data.Nat using ( ℕ )
module Data.PropFormula.Syntax ( n : ℕ ) where
------------------------------------------------------------------------------
open import Data.Bool
renaming ( _∧_ to _&&_; _∨_ to _||_ )
using ( Bool; true; false; not )
open import Data.Fin using ( Fin; #_ )
open import Data.List using ( List ; [] ; _∷_ ; _++_ ; [_] )
open import Relation.Binary.PropositionalEquality
using ( _≡_; refl; cong; trans; sym; subst)
------------------------------------------------------------------------------
-- Proposition data type.
data PropFormula : Set where
Var : Fin n → PropFormula
⊤ : PropFormula
⊥ : PropFormula
_∧_ _∨_ _⊃_ _⇔_ : (φ ψ : PropFormula) → PropFormula
¬_ : (φ : PropFormula) → PropFormula
infix 11 ¬_
infixl 8 _∧_ _∨_
infixr 7 _⊃_ _⇔_
-- Context is a list (set) of hypotesis and axioms.
Ctxt : Set
Ctxt = List PropFormula
infixl 5 _,_
_,_ : Ctxt → PropFormula → Ctxt
Γ , φ = Γ ++ [ φ ]
∅ : Ctxt
∅ = []
infix 30 _⨆_
_⨆_ : Ctxt → Ctxt → Ctxt
Γ ⨆ Δ = Γ ++ Δ
infix 4 _∈_
data _∈_ (φ : PropFormula) : Ctxt → Set where
here : ∀ {Γ} → φ ∈ Γ , φ
there : ∀ {Γ} → (ψ : PropFormula) → φ ∈ Γ → φ ∈ Γ , ψ
⨆-ext : ∀ {Γ} → (Δ : Ctxt) → φ ∈ Γ → φ ∈ Γ ⨆ Δ
_⊆_ : Ctxt → Ctxt → Set
Γ ⊆ Η = ∀ {φ} → φ ∈ Γ → φ ∈ Η
------------------------------------------------------------------------
-- Theorem data type.
infix 3 _⊢_
data _⊢_ : Ctxt → PropFormula → Set where
-- Hyp.
assume : ∀ {Γ} → (φ : PropFormula) → Γ , φ ⊢ φ
axiom : ∀ {Γ} → (φ : PropFormula) → φ ∈ Γ
→ Γ ⊢ φ
weaken : ∀ {Γ} {φ} → (ψ : PropFormula) → Γ ⊢ φ
→ Γ , ψ ⊢ φ
weaken₂ : ∀ {Γ} {φ} → (ψ : PropFormula) → Γ ⊢ φ
→ ψ ∷ Γ ⊢ φ
-- Top and Bottom.
⊤-intro : ∀ {Γ} → Γ ⊢ ⊤
⊥-elim : ∀ {Γ} → (φ : PropFormula) → Γ ⊢ ⊥
→ Γ ⊢ φ
-- Negation.
¬-intro : ∀ {Γ} {φ} → Γ , φ ⊢ ⊥
→ Γ ⊢ ¬ φ
¬-elim : ∀ {Γ} {φ} → Γ ⊢ ¬ φ → Γ ⊢ φ
→ Γ ⊢ ⊥
-- Conjunction.
∧-intro : ∀ {Γ} {φ ψ} → Γ ⊢ φ → Γ ⊢ ψ
→ Γ ⊢ φ ∧ ψ
∧-proj₁ : ∀ {Γ} {φ ψ} → Γ ⊢ φ ∧ ψ
→ Γ ⊢ φ
∧-proj₂ : ∀ {Γ} {φ ψ} → Γ ⊢ φ ∧ ψ
→ Γ ⊢ ψ
-- Disjunction.
∨-intro₁ : ∀ {Γ} {φ} → (ψ : PropFormula) → Γ ⊢ φ
→ Γ ⊢ φ ∨ ψ
∨-intro₂ : ∀ {Γ} {ψ} → (φ : PropFormula) → Γ ⊢ ψ
→ Γ ⊢ φ ∨ ψ
∨-elim : ∀ {Γ} {φ ψ χ} → Γ , φ ⊢ χ
→ Γ , ψ ⊢ χ
→ Γ , φ ∨ ψ ⊢ χ
-- Implication.
⊃-intro : ∀ {Γ} {φ ψ} → Γ , φ ⊢ ψ
→ Γ ⊢ φ ⊃ ψ
⊃-elim : ∀ {Γ} {φ ψ} → Γ ⊢ φ ⊃ ψ → Γ ⊢ φ
→ Γ ⊢ ψ
-- Biconditional.
⇔-intro : ∀ {Γ} {φ ψ} → Γ , φ ⊢ ψ
→ Γ , ψ ⊢ φ
→ Γ ⊢ φ ⇔ ψ
⇔-elim₁ : ∀ {Γ} {φ ψ} → Γ ⊢ φ → Γ ⊢ φ ⇔ ψ
→ Γ ⊢ ψ
⇔-elim₂ : ∀ {Γ} {φ ψ} → Γ ⊢ ψ → Γ ⊢ φ ⇔ ψ
→ Γ ⊢ φ
------------------------------------------------------------------------
| {
"alphanum_fraction": 0.282032032,
"avg_line_length": 30.045112782,
"ext": "agda",
"hexsha": "0abac0722add3fbfa8fefe5dca426fbdfaacd02c",
"lang": "Agda",
"max_forks_count": 2,
"max_forks_repo_forks_event_max_datetime": "2017-12-01T17:01:25.000Z",
"max_forks_repo_forks_event_min_datetime": "2017-03-30T16:41:56.000Z",
"max_forks_repo_head_hexsha": "a1730062a6aaced2bb74878c1071db06477044ae",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "jonaprieto/agda-prop",
"max_forks_repo_path": "src/Data/PropFormula/Syntax.agda",
"max_issues_count": 18,
"max_issues_repo_head_hexsha": "a1730062a6aaced2bb74878c1071db06477044ae",
"max_issues_repo_issues_event_max_datetime": "2017-12-18T16:34:21.000Z",
"max_issues_repo_issues_event_min_datetime": "2017-03-08T14:33:10.000Z",
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "jonaprieto/agda-prop",
"max_issues_repo_path": "src/Data/PropFormula/Syntax.agda",
"max_line_length": 78,
"max_stars_count": 13,
"max_stars_repo_head_hexsha": "a1730062a6aaced2bb74878c1071db06477044ae",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "jonaprieto/agda-prop",
"max_stars_repo_path": "src/Data/PropFormula/Syntax.agda",
"max_stars_repo_stars_event_max_datetime": "2022-01-17T03:33:12.000Z",
"max_stars_repo_stars_event_min_datetime": "2017-05-01T16:45:41.000Z",
"num_tokens": 1271,
"size": 3996
} |
{-# OPTIONS --safe #-} -- implies --no-sized-types
module Issue3517.M where
open import Issue3517.S
f : (i : Size) (j : Size< i) → Size< j → Size< i
f i j k = k
| {
"alphanum_fraction": 0.5975609756,
"avg_line_length": 18.2222222222,
"ext": "agda",
"hexsha": "cf1db2960a759d9a1e12bc4d0d2213e0a5b173ed",
"lang": "Agda",
"max_forks_count": 371,
"max_forks_repo_forks_event_max_datetime": "2022-03-30T19:00:30.000Z",
"max_forks_repo_forks_event_min_datetime": "2015-01-03T14:04:08.000Z",
"max_forks_repo_head_hexsha": "231d6ad8e77b67ff8c4b1cb35a6c31ccd988c3e9",
"max_forks_repo_licenses": [
"BSD-3-Clause"
],
"max_forks_repo_name": "Agda-zh/agda",
"max_forks_repo_path": "test/Fail/Issue3517/M.agda",
"max_issues_count": 4066,
"max_issues_repo_head_hexsha": "ed8ac6f4062ea8a20fa0f62d5db82d4e68278338",
"max_issues_repo_issues_event_max_datetime": "2022-03-31T21:14:49.000Z",
"max_issues_repo_issues_event_min_datetime": "2015-01-10T11:24:51.000Z",
"max_issues_repo_licenses": [
"BSD-3-Clause"
],
"max_issues_repo_name": "shlevy/agda",
"max_issues_repo_path": "test/Fail/Issue3517/M.agda",
"max_line_length": 50,
"max_stars_count": 1989,
"max_stars_repo_head_hexsha": "ed8ac6f4062ea8a20fa0f62d5db82d4e68278338",
"max_stars_repo_licenses": [
"BSD-3-Clause"
],
"max_stars_repo_name": "shlevy/agda",
"max_stars_repo_path": "test/Fail/Issue3517/M.agda",
"max_stars_repo_stars_event_max_datetime": "2022-03-30T18:20:48.000Z",
"max_stars_repo_stars_event_min_datetime": "2015-01-09T23:51:16.000Z",
"num_tokens": 57,
"size": 164
} |
module Models where
open import Data.Nat
open import Terms
-- The (complete) Herbrand universe for Σ
U' : {n m : ℕ} → (Signature n m) → Set
U' Σ = GTerm Σ
-- The (complete) μ-Herbrand base for Σ
B'μ : {n m : ℕ} → (Signature n m) → Set
B'μ Σ = GAtom Σ μ
B'ν : {n m : ℕ} → (Signature n m) → Set
B'ν Σ = GAtom Σ ν
open import Relation.Unary as U
open import Level
-- a (complete) Herbrand interpretation
record Interp {n m : ℕ} (Σ : Signature n m) : Set₁ where
field
Carrier-μ : Pred (B'μ Σ) Level.zero
Carrier-ν : Pred (B'ν Σ) Level.zero
open Interp
_∩ᵢ_ : {n m : ℕ} → {Σ : Signature n m} → Interp Σ → Interp Σ
→ Interp Σ
i₁ ∩ᵢ i₂ = record
{ Carrier-μ = Carrier-μ i₁ ∩ Carrier-μ i₂
; Carrier-ν = Carrier-ν i₁ ∩ Carrier-ν i₂
}
_∪ᵢ_ : {n m : ℕ} → {Σ : Signature n m} → Interp Σ → Interp Σ
→ Interp Σ
i₁ ∪ᵢ i₂ = record
{ Carrier-μ = Carrier-μ i₁ ∪ Carrier-μ i₂
; Carrier-ν = Carrier-ν i₁ ∪ Carrier-ν i₂
}
open import Data.List as L
open import Data.List.All as LAl
open import Data.List.Any as LAn
open import Relation.Binary.Core
open Program
-- | Inductive model
record IsIModel {n m : ℕ} {Σ : Signature n m} {var : Set}
(i : Interp Σ) (P : Program Σ var) : Set₂ where
field
forwClosed :
(bs'μ : List (GAtom Σ μ))
→ All (λ b → b ∈ Carrier-μ i) bs'μ
→ (bs'ν : List (GAtom Σ ν))
→ All (λ b → b ∈ Carrier-ν i) bs'ν
→ (σ : GSubst Σ var)
→ (a : Atom Σ var μ)
→ (bsμ : List (Atom Σ var μ))
→ (bsν : List (Atom Σ var ν))
→ Any (λ cl → cl ≡ (a :- bsμ , bsν)) (prg-μ P)
→ (L.map (appA σ) bsμ) ≡ bs'μ
→ (L.map (appA σ) bsν) ≡ bs'ν
→ (appA σ a ∈ Carrier-μ i)
open IsIModel
open import Data.Product
hA : {A : Set} {B : Set₁} → A × B → A
hA = proj₁
hBsμ : {A B : Set} {C : Set₁} → A × B × C → B
hBsμ (_ , a , _) = a
hBsν : {A B C : Set} {D : Set₁} → A × B × C × D → C
hBsν (_ , _ , a , _) = a
hσ : {A B C : Set} {D : Set₁} → A × B × C × D → D
hσ (_ , _ , _ , a) = a
open import Data.List.All.Properties -- using (All-map)
-- | model intersection property for a pair of models
prop_model_intersection_pair : {n m : ℕ} → {Σ : Signature n m} {var : Set} →
(P : Program Σ var)
→ (m₁ : Interp Σ)
→ (m₂ : Interp Σ)
→ Carrier-ν m₁ ≡ Carrier-ν m₂
→ (mp₁ : IsIModel m₁ P)
→ (mp₂ : IsIModel m₂ P)
→ IsIModel (m₁ ∩ᵢ m₂) P
prop_model_intersection_pair P m₁ m₂ eq mp₁ mp₂ =
record { forwClosed = λ bs'μ x bs'ν y σ a bsμ bsν pcls pμ pν →
( forwClosed mp₁ bs'μ (LAl.map proj₁ x) bs'ν
(LAl.map proj₁ y) σ a bsμ bsν pcls pμ pν
, forwClosed mp₂ bs'μ (LAl.map proj₂ x) bs'ν
(LAl.map proj₂ y) σ a bsμ bsν pcls pμ pν
)}
-- | Coinductive model
record IsCModel {n m : ℕ} {Σ : Signature n m} {var : Set}
(i : Interp Σ) (P : Program Σ var) : Set₁ where
field
backClosed :
--→
(a' : GAtom Σ ν)
→ a' ∈ Carrier-ν i
→ ∃ (λ ( w : (Atom Σ var ν) -- a
× (List (Atom Σ var μ)) -- bs-μ
× (List (Atom Σ var ν)) -- bs-ν
× GSubst Σ var) → -- σ
(Any (λ c → (hA w) :- (hBsμ w) , (hBsν w) ≡ c) (prg-ν P))
× appA (hσ w) (hA w) ≡ a'
× All (λ c → c ∈ Carrier-μ i) (L.map (appA (hσ w)) (hBsμ w))
× All (λ c → c ∈ Carrier-ν i) (L.map (appA (hσ w)) (hBsν w))
)
open IsCModel
open import Data.Sum
open import Data.Product as DP
open Interp
open import Relation.Binary.PropositionalEquality
-- | model union property for a pair of models
prop_model_union_pair : {n m : ℕ} → {Σ : Signature n m} → {var : Set}
(P : Program Σ var)
→ (m₁ : Interp Σ)
→ (m₂ : Interp Σ)
→ Carrier-μ m₁ ≡ Carrier-μ m₂
→ (mp₁ : IsCModel m₁ P)
→ (mp₂ : IsCModel m₂ P)
→ IsCModel (m₁ ∪ᵢ m₂) P
prop_model_union_pair P m₁ m₂ eq mp₁ mp₂ {-with (sym eq) -- | (Carrier-μ m₁)
... | eq' {-| dm₁-}-} = record { backClosed = λ
{ a' (inj₁ x) → DP.map
(λ atm → atm)
(DP.map
(λ any → any)
(λ w → DP.map (λ eq₁ → eq₁) (λ x₃
→ LAl.map inj₁ (proj₁ (proj₂ w))
, LAl.map inj₁ (proj₂ (proj₂ w))) w))
(backClosed mp₁ a' x)
; a' (inj₂ y) → DP.map
(λ atm → atm)
(DP.map
(λ any → any)
(λ w → DP.map (λ eq → eq) (λ x₁
→ LAl.map inj₂ (proj₁ (proj₂ w))
, LAl.map inj₂ (proj₂ (proj₂ w))) w))
(backClosed mp₂ a' y)
} }
| {
"alphanum_fraction": 0.5368589744,
"avg_line_length": 27.4716981132,
"ext": "agda",
"hexsha": "97780aace4557a2859ff974eeed25b91bbbece88",
"lang": "Agda",
"max_forks_count": null,
"max_forks_repo_forks_event_max_datetime": null,
"max_forks_repo_forks_event_min_datetime": null,
"max_forks_repo_head_hexsha": "411ca7970b6f64857a36ebcf648c9a58b90bb4b2",
"max_forks_repo_licenses": [
"BSD-2-Clause"
],
"max_forks_repo_name": "frantisekfarka/lp-mod",
"max_forks_repo_path": "Mixed/Models.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "411ca7970b6f64857a36ebcf648c9a58b90bb4b2",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"BSD-2-Clause"
],
"max_issues_repo_name": "frantisekfarka/lp-mod",
"max_issues_repo_path": "Mixed/Models.agda",
"max_line_length": 76,
"max_stars_count": null,
"max_stars_repo_head_hexsha": "411ca7970b6f64857a36ebcf648c9a58b90bb4b2",
"max_stars_repo_licenses": [
"BSD-2-Clause"
],
"max_stars_repo_name": "frantisekfarka/lp-mod",
"max_stars_repo_path": "Mixed/Models.agda",
"max_stars_repo_stars_event_max_datetime": null,
"max_stars_repo_stars_event_min_datetime": null,
"num_tokens": 1780,
"size": 4368
} |
------------------------------------------------------------------------
-- The Agda standard library
--
-- Primitive IO: simple bindings to Haskell types and functions
------------------------------------------------------------------------
module IO.Primitive where
open import Data.Char
open import Data.String
open import Foreign.Haskell
------------------------------------------------------------------------
-- The IO monad
postulate
IO : ∀ {ℓ} → Set ℓ → Set ℓ
{-# IMPORT IO.FFI #-}
{-# COMPILED_TYPE IO IO.FFI.AgdaIO #-}
{-# BUILTIN IO IO #-}
infixl 1 _>>=_
postulate
return : ∀ {a} {A : Set a} → A → IO A
_>>=_ : ∀ {a b} {A : Set a} {B : Set b} → IO A → (A → IO B) → IO B
{-# COMPILED return (\_ _ -> return) #-}
{-# COMPILED _>>=_ (\_ _ _ _ -> (>>=)) #-}
------------------------------------------------------------------------
-- Simple lazy IO
-- Note that the functions below produce commands which, when
-- executed, may raise exceptions.
-- Note also that the semantics of these functions depends on the
-- version of the Haskell base library. If the version is 4.2.0.0 (or
-- later?), then the functions use the character encoding specified by
-- the locale. For older versions of the library (going back to at
-- least version 3) the functions use ISO-8859-1.
postulate
getContents : IO Costring
readFile : String → IO Costring
writeFile : String → Costring → IO Unit
appendFile : String → Costring → IO Unit
putStr : Costring → IO Unit
putStrLn : Costring → IO Unit
-- Reads a finite file. Raises an exception if the file path refers
-- to a non-physical file (like "/dev/zero").
readFiniteFile : String → IO String
{-# COMPILED getContents getContents #-}
{-# COMPILED readFile readFile #-}
{-# COMPILED writeFile writeFile #-}
{-# COMPILED appendFile appendFile #-}
{-# COMPILED putStr putStr #-}
{-# COMPILED putStrLn putStrLn #-}
{-# COMPILED readFiniteFile IO.FFI.readFiniteFile #-}
| {
"alphanum_fraction": 0.5391304348,
"avg_line_length": 32.34375,
"ext": "agda",
"hexsha": "e45542530e574e4eda84dbeb58908a3463aa9087",
"lang": "Agda",
"max_forks_count": null,
"max_forks_repo_forks_event_max_datetime": null,
"max_forks_repo_forks_event_min_datetime": null,
"max_forks_repo_head_hexsha": "9d4c43b1609d3f085636376fdca73093481ab882",
"max_forks_repo_licenses": [
"Apache-2.0"
],
"max_forks_repo_name": "qwe2/try-agda",
"max_forks_repo_path": "agda-stdlib-0.9/src/IO/Primitive.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "9d4c43b1609d3f085636376fdca73093481ab882",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"Apache-2.0"
],
"max_issues_repo_name": "qwe2/try-agda",
"max_issues_repo_path": "agda-stdlib-0.9/src/IO/Primitive.agda",
"max_line_length": 72,
"max_stars_count": 1,
"max_stars_repo_head_hexsha": "9d4c43b1609d3f085636376fdca73093481ab882",
"max_stars_repo_licenses": [
"Apache-2.0"
],
"max_stars_repo_name": "qwe2/try-agda",
"max_stars_repo_path": "agda-stdlib-0.9/src/IO/Primitive.agda",
"max_stars_repo_stars_event_max_datetime": "2016-10-20T15:52:05.000Z",
"max_stars_repo_stars_event_min_datetime": "2016-10-20T15:52:05.000Z",
"num_tokens": 488,
"size": 2070
} |
------------------------------------------------------------------------
-- The Agda standard library
--
-- Dependent product combinators for propositional equality
-- preserving functions
------------------------------------------------------------------------
{-# OPTIONS --without-K --safe #-}
module Data.Product.Function.Dependent.Propositional where
open import Data.Product
open import Data.Product.Function.NonDependent.Setoid
open import Data.Product.Relation.Binary.Pointwise.NonDependent
open import Relation.Binary
open import Function
open import Function.Equality using (_⟶_; _⟨$⟩_)
open import Function.Equivalence as Equiv using (_⇔_; module Equivalence)
open import Function.HalfAdjointEquivalence using (↔→≃; _≃_)
open import Function.Injection as Inj
using (Injective; _↣_; module Injection)
open import Function.Inverse as Inv using (_↔_; module Inverse)
open import Function.LeftInverse as LeftInv
using (_↞_; _LeftInverseOf_; module LeftInverse)
open import Function.Related
open import Function.Related.TypeIsomorphisms
open import Function.Surjection as Surj using (_↠_; module Surjection)
open import Relation.Binary.PropositionalEquality as P using (_≡_)
------------------------------------------------------------------------
-- Combinators for various function types
module _ {a₁ a₂} {A₁ : Set a₁} {A₂ : Set a₂}
{b₁ b₂} {B₁ : A₁ → Set b₁} {B₂ : A₂ → Set b₂}
where
⇔ : (A₁⇔A₂ : A₁ ⇔ A₂) →
(∀ {x} → B₁ x → B₂ (Equivalence.to A₁⇔A₂ ⟨$⟩ x)) →
(∀ {y} → B₂ y → B₁ (Equivalence.from A₁⇔A₂ ⟨$⟩ y)) →
Σ A₁ B₁ ⇔ Σ A₂ B₂
⇔ A₁⇔A₂ B-to B-from = Equiv.equivalence
(map (Equivalence.to A₁⇔A₂ ⟨$⟩_) B-to)
(map (Equivalence.from A₁⇔A₂ ⟨$⟩_) B-from)
⇔-↠ : ∀ (A₁↠A₂ : A₁ ↠ A₂) →
(∀ {x} → _⇔_ (B₁ x) (B₂ (Surjection.to A₁↠A₂ ⟨$⟩ x))) →
_⇔_ (Σ A₁ B₁) (Σ A₂ B₂)
⇔-↠ A₁↠A₂ B₁⇔B₂ = Equiv.equivalence
(map (Surjection.to A₁↠A₂ ⟨$⟩_) (Equivalence.to B₁⇔B₂ ⟨$⟩_))
(map (Surjection.from A₁↠A₂ ⟨$⟩_)
((Equivalence.from B₁⇔B₂ ⟨$⟩_) ∘
P.subst B₂ (P.sym $ Surjection.right-inverse-of A₁↠A₂ _)))
-- See also Data.Product.Relation.Binary.Pointwise.Dependent.WithK.↣.
↣ : ∀ (A₁↔A₂ : A₁ ↔ A₂) →
(∀ {x} → B₁ x ↣ B₂ (Inverse.to A₁↔A₂ ⟨$⟩ x)) →
Σ A₁ B₁ ↣ Σ A₂ B₂
↣ A₁↔A₂ B₁↣B₂ = Inj.injection to to-injective
where
open P.≡-Reasoning
A₁≃A₂ = ↔→≃ A₁↔A₂
subst-application′ :
let open _≃_ A₁≃A₂ in
{x₁ x₂ : A₁} {y : B₁ (from (to x₁))}
(g : ∀ x → B₁ (from (to x)) → B₂ (to x)) (eq : to x₁ ≡ to x₂) →
P.subst B₂ eq (g x₁ y) ≡ g x₂ (P.subst B₁ (P.cong from eq) y)
subst-application′ {x₁} {x₂} {y} g eq =
P.subst B₂ eq (g x₁ y) ≡⟨ P.cong (P.subst B₂ eq) (P.sym (g′-lemma _ _)) ⟩
P.subst B₂ eq (g′ (to x₁) y) ≡⟨ P.subst-application B₁ g′ eq ⟩
g′ (to x₂) (P.subst B₁ (P.cong from eq) y) ≡⟨ g′-lemma _ _ ⟩
g x₂ (P.subst B₁ (P.cong from eq) y) ∎
where
open _≃_ A₁≃A₂
g′ : ∀ x → B₁ (from x) → B₂ x
g′ x =
P.subst B₂ (right-inverse-of x) ∘
g (from x) ∘
P.subst B₁ (P.sym (P.cong from (right-inverse-of x)))
g′-lemma : ∀ x y → g′ (to x) y ≡ g x y
g′-lemma x y =
P.subst B₂ (right-inverse-of (to x))
(g (from (to x)) $
P.subst B₁ (P.sym (P.cong from (right-inverse-of (to x)))) y) ≡⟨ P.cong (λ p → P.subst B₂ p (g (from (to x))
(P.subst B₁ (P.sym (P.cong from p)) y)))
(P.sym (left-right x)) ⟩
P.subst B₂ (P.cong to (left-inverse-of x))
(g (from (to x)) $
P.subst B₁
(P.sym (P.cong from (P.cong to (left-inverse-of x))))
y) ≡⟨ lemma _ ⟩
g x y ∎
where
lemma :
∀ {x′} eq {y : B₁ (from (to x′))} →
P.subst B₂ (P.cong to eq)
(g (from (to x))
(P.subst B₁ (P.sym (P.cong from (P.cong to eq))) y)) ≡
g x′ y
lemma P.refl = P.refl
to = map (_≃_.to A₁≃A₂) (Injection.to B₁↣B₂ ⟨$⟩_)
to-injective : Injective (P.→-to-⟶ {B = P.setoid _} to)
to-injective {(x₁ , x₂)} {(y₁ , y₂)} =
(Inverse.to Σ-≡,≡↔≡ ⟨$⟩_) ∘′
map (_≃_.injective A₁≃A₂) (λ {eq₁} eq₂ →
let lemma =
Injection.to B₁↣B₂ ⟨$⟩
P.subst B₁ (_≃_.injective A₁≃A₂ eq₁) x₂ ≡⟨⟩
Injection.to B₁↣B₂ ⟨$⟩
P.subst B₁
(P.trans (P.sym (_≃_.left-inverse-of A₁≃A₂ x₁))
(P.trans (P.cong (_≃_.from A₁≃A₂) eq₁)
(P.trans (_≃_.left-inverse-of A₁≃A₂ y₁)
P.refl)))
x₂ ≡⟨ P.cong (λ p → Injection.to B₁↣B₂ ⟨$⟩
P.subst B₁
(P.trans (P.sym (_≃_.left-inverse-of A₁≃A₂ _))
(P.trans (P.cong (_≃_.from A₁≃A₂) eq₁) p))
x₂)
(P.trans-reflʳ _) ⟩
Injection.to B₁↣B₂ ⟨$⟩
P.subst B₁
(P.trans (P.sym (_≃_.left-inverse-of A₁≃A₂ x₁))
(P.trans (P.cong (_≃_.from A₁≃A₂) eq₁)
(_≃_.left-inverse-of A₁≃A₂ y₁)))
x₂ ≡⟨ P.cong (Injection.to B₁↣B₂ ⟨$⟩_)
(P.sym (P.subst-subst (P.sym (_≃_.left-inverse-of A₁≃A₂ _)))) ⟩
Injection.to B₁↣B₂ ⟨$⟩
(P.subst B₁ (P.trans (P.cong (_≃_.from A₁≃A₂) eq₁)
(_≃_.left-inverse-of A₁≃A₂ y₁)) $
P.subst B₁ (P.sym (_≃_.left-inverse-of A₁≃A₂ x₁)) x₂) ≡⟨ P.cong (Injection.to B₁↣B₂ ⟨$⟩_)
(P.sym (P.subst-subst (P.cong (_≃_.from A₁≃A₂) eq₁))) ⟩
Injection.to B₁↣B₂ ⟨$⟩
(P.subst B₁ (_≃_.left-inverse-of A₁≃A₂ y₁) $
P.subst B₁ (P.cong (_≃_.from A₁≃A₂) eq₁) $
P.subst B₁ (P.sym (_≃_.left-inverse-of A₁≃A₂ x₁)) x₂) ≡⟨ P.sym (subst-application′
(λ x y → Injection.to B₁↣B₂ ⟨$⟩
P.subst B₁ (_≃_.left-inverse-of A₁≃A₂ x) y)
eq₁) ⟩
P.subst B₂ eq₁
(Injection.to B₁↣B₂ ⟨$⟩
(P.subst B₁ (_≃_.left-inverse-of A₁≃A₂ x₁) $
P.subst B₁ (P.sym (_≃_.left-inverse-of A₁≃A₂ x₁)) x₂)) ≡⟨ P.cong (P.subst B₂ eq₁ ∘ (Injection.to B₁↣B₂ ⟨$⟩_))
(P.subst-subst (P.sym (_≃_.left-inverse-of A₁≃A₂ _))) ⟩
P.subst B₂ eq₁
(Injection.to B₁↣B₂ ⟨$⟩
P.subst B₁
(P.trans (P.sym (_≃_.left-inverse-of A₁≃A₂ x₁))
(_≃_.left-inverse-of A₁≃A₂ x₁))
x₂) ≡⟨ P.cong (λ p → P.subst B₂ eq₁
(Injection.to B₁↣B₂ ⟨$⟩ P.subst B₁ p x₂))
(P.trans-symˡ (_≃_.left-inverse-of A₁≃A₂ _)) ⟩
P.subst B₂ eq₁
(Injection.to B₁↣B₂ ⟨$⟩ P.subst B₁ P.refl x₂) ≡⟨⟩
P.subst B₂ eq₁ (Injection.to B₁↣B₂ ⟨$⟩ x₂) ≡⟨ eq₂ ⟩
Injection.to B₁↣B₂ ⟨$⟩ y₂ ∎
in
P.subst B₁ (_≃_.injective A₁≃A₂ eq₁) x₂ ≡⟨ Injection.injective B₁↣B₂ lemma ⟩
y₂ ∎) ∘
(Inverse.from Σ-≡,≡↔≡ ⟨$⟩_)
↞ : (A₁↞A₂ : A₁ ↞ A₂) →
(∀ {x} → B₁ (LeftInverse.from A₁↞A₂ ⟨$⟩ x) ↞ B₂ x) →
Σ A₁ B₁ ↞ Σ A₂ B₂
↞ A₁↞A₂ B₁↞B₂ = record
{ to = P.→-to-⟶ to
; from = P.→-to-⟶ from
; left-inverse-of = left-inverse-of
}
where
open P.≡-Reasoning
from = map (LeftInverse.from A₁↞A₂ ⟨$⟩_) (LeftInverse.from B₁↞B₂ ⟨$⟩_)
to = map
(LeftInverse.to A₁↞A₂ ⟨$⟩_)
(λ {x} y →
LeftInverse.to B₁↞B₂ ⟨$⟩
P.subst B₁ (P.sym (LeftInverse.left-inverse-of A₁↞A₂ x)) y)
left-inverse-of : ∀ p → from (to p) ≡ p
left-inverse-of (x , y) = Inverse.to Σ-≡,≡↔≡ ⟨$⟩
( LeftInverse.left-inverse-of A₁↞A₂ x
, (P.subst B₁ (LeftInverse.left-inverse-of A₁↞A₂ x)
(LeftInverse.from B₁↞B₂ ⟨$⟩ (LeftInverse.to B₁↞B₂ ⟨$⟩
(P.subst B₁ (P.sym (LeftInverse.left-inverse-of A₁↞A₂ x))
y))) ≡⟨ P.cong (P.subst B₁ _) (LeftInverse.left-inverse-of B₁↞B₂ _) ⟩
P.subst B₁ (LeftInverse.left-inverse-of A₁↞A₂ x)
(P.subst B₁ (P.sym (LeftInverse.left-inverse-of A₁↞A₂ x))
y) ≡⟨ P.subst-subst-sym (LeftInverse.left-inverse-of A₁↞A₂ x) ⟩
y ∎)
)
↠ : (A₁↠A₂ : A₁ ↠ A₂) →
(∀ {x} → B₁ x ↠ B₂ (Surjection.to A₁↠A₂ ⟨$⟩ x)) →
Σ A₁ B₁ ↠ Σ A₂ B₂
↠ A₁↠A₂ B₁↠B₂ = record
{ to = P.→-to-⟶ to
; surjective = record
{ from = P.→-to-⟶ from
; right-inverse-of = right-inverse-of
}
}
where
open P.≡-Reasoning
to = map (Surjection.to A₁↠A₂ ⟨$⟩_)
(Surjection.to B₁↠B₂ ⟨$⟩_)
from = map
(Surjection.from A₁↠A₂ ⟨$⟩_)
(λ {x} y →
Surjection.from B₁↠B₂ ⟨$⟩
P.subst B₂ (P.sym (Surjection.right-inverse-of A₁↠A₂ x)) y)
right-inverse-of : ∀ p → to (from p) ≡ p
right-inverse-of (x , y) = Inverse.to Σ-≡,≡↔≡ ⟨$⟩
( Surjection.right-inverse-of A₁↠A₂ x
, (P.subst B₂ (Surjection.right-inverse-of A₁↠A₂ x)
(Surjection.to B₁↠B₂ ⟨$⟩ (Surjection.from B₁↠B₂ ⟨$⟩
(P.subst B₂ (P.sym (Surjection.right-inverse-of A₁↠A₂ x))
y))) ≡⟨ P.cong (P.subst B₂ _) (Surjection.right-inverse-of B₁↠B₂ _) ⟩
P.subst B₂ (Surjection.right-inverse-of A₁↠A₂ x)
(P.subst B₂ (P.sym (Surjection.right-inverse-of A₁↠A₂ x))
y) ≡⟨ P.subst-subst-sym (Surjection.right-inverse-of A₁↠A₂ x) ⟩
y ∎)
)
↔ : (A₁↔A₂ : A₁ ↔ A₂) →
(∀ {x} → B₁ x ↔ B₂ (Inverse.to A₁↔A₂ ⟨$⟩ x)) →
Σ A₁ B₁ ↔ Σ A₂ B₂
↔ A₁↔A₂ B₁↔B₂ = Inv.inverse
(Surjection.to surjection′ ⟨$⟩_)
(Surjection.from surjection′ ⟨$⟩_)
left-inverse-of
(Surjection.right-inverse-of surjection′)
where
open P.≡-Reasoning
A₁≃A₂ = ↔→≃ A₁↔A₂
surjection′ : _↠_ (Σ A₁ B₁) (Σ A₂ B₂)
surjection′ =
↠ (Inverse.surjection (_≃_.inverse A₁≃A₂))
(Inverse.surjection B₁↔B₂)
left-inverse-of :
∀ p → Surjection.from surjection′ ⟨$⟩
(Surjection.to surjection′ ⟨$⟩ p) ≡ p
left-inverse-of (x , y) = Inverse.to Σ-≡,≡↔≡ ⟨$⟩
( _≃_.left-inverse-of A₁≃A₂ x
, (P.subst B₁ (_≃_.left-inverse-of A₁≃A₂ x)
(Inverse.from B₁↔B₂ ⟨$⟩
(P.subst B₂ (P.sym (_≃_.right-inverse-of A₁≃A₂
(_≃_.to A₁≃A₂ x)))
(Inverse.to B₁↔B₂ ⟨$⟩ y))) ≡⟨ P.subst-application B₂ (λ _ → Inverse.from B₁↔B₂ ⟨$⟩_) _ ⟩
Inverse.from B₁↔B₂ ⟨$⟩
(P.subst B₂ (P.cong (_≃_.to A₁≃A₂)
(_≃_.left-inverse-of A₁≃A₂ x))
(P.subst B₂ (P.sym (_≃_.right-inverse-of A₁≃A₂
(_≃_.to A₁≃A₂ x)))
(Inverse.to B₁↔B₂ ⟨$⟩ y))) ≡⟨ P.cong (λ eq → Inverse.from B₁↔B₂ ⟨$⟩ P.subst B₂ eq
(P.subst B₂ (P.sym (_≃_.right-inverse-of A₁≃A₂ _)) _))
(_≃_.left-right A₁≃A₂ _) ⟩
Inverse.from B₁↔B₂ ⟨$⟩
(P.subst B₂ (_≃_.right-inverse-of A₁≃A₂
(_≃_.to A₁≃A₂ x))
(P.subst B₂ (P.sym (_≃_.right-inverse-of A₁≃A₂
(_≃_.to A₁≃A₂ x)))
(Inverse.to B₁↔B₂ ⟨$⟩ y))) ≡⟨ P.cong (Inverse.from B₁↔B₂ ⟨$⟩_)
(P.subst-subst-sym (_≃_.right-inverse-of A₁≃A₂ _)) ⟩
Inverse.from B₁↔B₂ ⟨$⟩ (Inverse.to B₁↔B₂ ⟨$⟩ y) ≡⟨ Inverse.left-inverse-of B₁↔B₂ _ ⟩
y ∎)
)
private
swap-coercions : ∀ {k a₁ a₂ b₁ b₂} {A₁ : Set a₁} {A₂ : Set a₂}
{B₁ : A₁ → Set b₁} (B₂ : A₂ → Set b₂)
(A₁↔A₂ : _↔_ A₁ A₂) →
(∀ {x} → B₁ x ∼[ k ] B₂ (Inverse.to A₁↔A₂ ⟨$⟩ x)) →
∀ {x} → B₁ (Inverse.from A₁↔A₂ ⟨$⟩ x) ∼[ k ] B₂ x
swap-coercions {k} {B₁ = B₁} B₂ A₁↔A₂ eq {x} =
B₁ (Inverse.from A₁↔A₂ ⟨$⟩ x)
∼⟨ eq ⟩
B₂ (Inverse.to A₁↔A₂ ⟨$⟩ (Inverse.from A₁↔A₂ ⟨$⟩ x))
↔⟨ K-reflexive
(P.cong B₂ $ Inverse.right-inverse-of A₁↔A₂ x) ⟩
B₂ x
∎
where open EquationalReasoning
cong : ∀ {k a₁ a₂ b₁ b₂}
{A₁ : Set a₁} {A₂ : Set a₂}
{B₁ : A₁ → Set b₁} {B₂ : A₂ → Set b₂}
(A₁↔A₂ : _↔_ A₁ A₂) →
(∀ {x} → B₁ x ∼[ k ] B₂ (Inverse.to A₁↔A₂ ⟨$⟩ x)) →
Σ A₁ B₁ ∼[ k ] Σ A₂ B₂
cong {implication} =
λ A₁↔A₂ → map (_⟨$⟩_ (Inverse.to A₁↔A₂))
cong {reverse-implication} {B₂ = B₂} =
λ A₁↔A₂ B₁←B₂ → lam (map (_⟨$⟩_ (Inverse.from A₁↔A₂))
(app-← (swap-coercions B₂ A₁↔A₂ B₁←B₂)))
cong {equivalence} = ⇔-↠ ∘ Inverse.surjection
cong {injection} = ↣
cong {reverse-injection} {B₂ = B₂} =
λ A₁↔A₂ B₁↢B₂ → lam (↣ (Inv.sym A₁↔A₂)
(app-↢ (swap-coercions B₂ A₁↔A₂ B₁↢B₂)))
cong {left-inverse} =
λ A₁↔A₂ → ↞ (Inverse.left-inverse A₁↔A₂) ∘ swap-coercions _ A₁↔A₂
cong {surjection} = ↠ ∘ Inverse.surjection
cong {bijection} = ↔
| {
"alphanum_fraction": 0.4206042859,
"avg_line_length": 44.8537313433,
"ext": "agda",
"hexsha": "746f73177a00a59d8f69ebab2f80e197a8f4a816",
"lang": "Agda",
"max_forks_count": null,
"max_forks_repo_forks_event_max_datetime": null,
"max_forks_repo_forks_event_min_datetime": null,
"max_forks_repo_head_hexsha": "0debb886eb5dbcd38dbeebd04b34cf9d9c5e0e71",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "omega12345/agda-mode",
"max_forks_repo_path": "test/asset/agda-stdlib-1.0/Data/Product/Function/Dependent/Propositional.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "0debb886eb5dbcd38dbeebd04b34cf9d9c5e0e71",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "omega12345/agda-mode",
"max_issues_repo_path": "test/asset/agda-stdlib-1.0/Data/Product/Function/Dependent/Propositional.agda",
"max_line_length": 147,
"max_stars_count": null,
"max_stars_repo_head_hexsha": "0debb886eb5dbcd38dbeebd04b34cf9d9c5e0e71",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "omega12345/agda-mode",
"max_stars_repo_path": "test/asset/agda-stdlib-1.0/Data/Product/Function/Dependent/Propositional.agda",
"max_stars_repo_stars_event_max_datetime": null,
"max_stars_repo_stars_event_min_datetime": null,
"num_tokens": 5218,
"size": 15026
} |
-- Andreas, 2018-07-22, issue #3136
-- WAS: Internal error when printing termination errors
{-# OPTIONS --postfix-projections #-}
module Issue3136 (A : Set) where
-- postulate A : Set
postulate
any : {X : Set} → X
x : A
P : A → Set
record C : Set where
field
a : A
b : P a
c : C
c = λ where
.C.a → x
.C.b → λ where
→ any
-- Should report a termination error but not crash
| {
"alphanum_fraction": 0.6044776119,
"avg_line_length": 15.4615384615,
"ext": "agda",
"hexsha": "3ab77d06dc6fc27b19e56ce0d8797c45cfcd5bd8",
"lang": "Agda",
"max_forks_count": 1,
"max_forks_repo_forks_event_max_datetime": "2021-04-01T18:30:09.000Z",
"max_forks_repo_forks_event_min_datetime": "2021-04-01T18:30:09.000Z",
"max_forks_repo_head_hexsha": "231d6ad8e77b67ff8c4b1cb35a6c31ccd988c3e9",
"max_forks_repo_licenses": [
"BSD-3-Clause"
],
"max_forks_repo_name": "Agda-zh/agda",
"max_forks_repo_path": "test/Fail/Issue3136.agda",
"max_issues_count": 3,
"max_issues_repo_head_hexsha": "aac88412199dd4cbcb041aab499d8a6b7e3f4a2e",
"max_issues_repo_issues_event_max_datetime": "2019-04-01T19:39:26.000Z",
"max_issues_repo_issues_event_min_datetime": "2018-11-14T15:31:44.000Z",
"max_issues_repo_licenses": [
"BSD-3-Clause"
],
"max_issues_repo_name": "hborum/agda",
"max_issues_repo_path": "test/Fail/Issue3136.agda",
"max_line_length": 55,
"max_stars_count": 2,
"max_stars_repo_head_hexsha": "aac88412199dd4cbcb041aab499d8a6b7e3f4a2e",
"max_stars_repo_licenses": [
"BSD-3-Clause"
],
"max_stars_repo_name": "hborum/agda",
"max_stars_repo_path": "test/Fail/Issue3136.agda",
"max_stars_repo_stars_event_max_datetime": "2020-09-20T00:28:57.000Z",
"max_stars_repo_stars_event_min_datetime": "2019-10-29T09:40:30.000Z",
"num_tokens": 136,
"size": 402
} |
{-# OPTIONS --with-K #-}
open import Agda.Builtin.Equality
open import Agda.Builtin.Nat
single : {m n : Nat} → suc m ≡ suc n → n ≡ m
single p with refl ← p = refl
double : {m n p : Nat} → suc m ≡ n → suc n ≡ 2 + p → m ≡ p
double p q with refl ← p | refl ← q = refl
_∋_ : (A : Set) → A → A
A ∋ a = a
-- The second equality proof is only well-typed
-- after the first one has been used
tele : {m n : Nat} → suc m ≡ suc n → m ≡ n
tele {m} {n} p
with refl ← p
with refl ← (n ≡ m) ∋ refl
= refl
tele' : {m n : Nat} → m ≡ n → m ≡ n
tele' {m} {n} p with refl ← p with (n ≡ m) ∋ refl
... | q = refl
-- Further splitting after a using & with
tele'' : {m n : Nat} → m ≡ n → Nat → Nat
tele'' {m} {n} p r with refl ← p | (n ≡ m) ∋ refl
tele'' {m} {m} p zero | q = m
tele'' {m} {m} p (suc r) | q = r
data Vec {a} (A : Set a) : Nat → Set a where
[] : Vec A 0
_∷_ : ∀ {n} → A → Vec A n → Vec A (suc n)
module _ {a} {A : Set a} {n} where
head : Vec A (suc n) → A
head xs with (x ∷ _) ← xs = x
tail : Vec A (suc n) → Vec A n
tail xs with (_ ∷ xs) ← xs = xs -- pattern shadows variable with'd on
castVec : ∀ {m n} → m ≡ n → Vec Nat m → Vec Nat n
castVec eq ms with refl ← eq = ms
data All (P : Nat → Set) : ∀ {n} → Vec Nat n → Set where
[] : All P []
_∷_ : ∀ {n x xs} → P x → All P {n} xs → All P (x ∷ xs)
open import Agda.Builtin.Sigma
castAll : ∀ {P m n xs ys} → Σ (m ≡ n) (λ eq → castVec eq xs ≡ ys) →
All P xs → All P ys
castAll (refl , refl) all = all
-- faking rewrite with the dependent irrefutable with
postulate +-comm : ∀ m n → m + n ≡ n + m
rew : ∀ m n p q → m + (p + q) + n ≡ m + (q + p) + n
rew m n p q with p+q ← p + q | refl ← +-comm p q {- : p + q ≡ q + p -} = refl
-- Note that the following does not work because
-- p+q is not abstracted over in `+-comm p q` which means
-- Agda gets stuck trying to unify `p + q` and `q + p`
-- Cf. test/Fail/UsingEq.agda
-- rew' : ∀ m n p q → m + (p + q) + n ≡ m + (q + p) + n
-- rew' m n p q with p+q ← p + q with refl ← +-comm p q = refl
| {
"alphanum_fraction": 0.5242766062,
"avg_line_length": 27.5540540541,
"ext": "agda",
"hexsha": "467fd8981c7103ec75b1597e9e717cf5d78002e2",
"lang": "Agda",
"max_forks_count": 371,
"max_forks_repo_forks_event_max_datetime": "2022-03-30T19:00:30.000Z",
"max_forks_repo_forks_event_min_datetime": "2015-01-03T14:04:08.000Z",
"max_forks_repo_head_hexsha": "7f58030124fa99dfbf8db376659416f3ad8384de",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "cruhland/agda",
"max_forks_repo_path": "test/Succeed/UsingEq.agda",
"max_issues_count": 4066,
"max_issues_repo_head_hexsha": "7f58030124fa99dfbf8db376659416f3ad8384de",
"max_issues_repo_issues_event_max_datetime": "2022-03-31T21:14:49.000Z",
"max_issues_repo_issues_event_min_datetime": "2015-01-10T11:24:51.000Z",
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "cruhland/agda",
"max_issues_repo_path": "test/Succeed/UsingEq.agda",
"max_line_length": 77,
"max_stars_count": 1989,
"max_stars_repo_head_hexsha": "7f58030124fa99dfbf8db376659416f3ad8384de",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "cruhland/agda",
"max_stars_repo_path": "test/Succeed/UsingEq.agda",
"max_stars_repo_stars_event_max_datetime": "2022-03-30T18:20:48.000Z",
"max_stars_repo_stars_event_min_datetime": "2015-01-09T23:51:16.000Z",
"num_tokens": 829,
"size": 2039
} |
------------------------------------------------------------------------
-- The Agda standard library
--
-- Divisibility
------------------------------------------------------------------------
{-# OPTIONS --without-K --safe #-}
module Data.Nat.Divisibility where
open import Algebra
open import Data.Nat.Base
open import Data.Nat.DivMod
open import Data.Nat.Properties
open import Data.Product
open import Function.Base
open import Function.Equivalence using (_⇔_; equivalence)
open import Level using (0ℓ)
open import Relation.Nullary using (yes; no)
open import Relation.Nullary.Decidable as Dec using (False)
open import Relation.Nullary.Negation using (contradiction)
open import Relation.Binary
import Relation.Binary.Reasoning.Preorder as PreorderReasoning
open import Relation.Binary.PropositionalEquality as PropEq
using (_≡_; _≢_; refl; sym; trans; cong; cong₂; subst)
------------------------------------------------------------------------
-- Definition
open import Data.Nat.Divisibility.Core public
------------------------------------------------------------------------
-- Relationship with _%_
m%n≡0⇒n∣m : ∀ m n → m % suc n ≡ 0 → suc n ∣ m
m%n≡0⇒n∣m m n eq = divides (m / suc n) (begin-equality
m ≡⟨ m≡m%n+[m/n]*n m n ⟩
m % suc n + m / suc n * (suc n) ≡⟨ cong₂ _+_ eq refl ⟩
m / suc n * (suc n) ∎)
where open ≤-Reasoning
n∣m⇒m%n≡0 : ∀ m n → suc n ∣ m → m % suc n ≡ 0
n∣m⇒m%n≡0 m n (divides v eq) = begin-equality
m % suc n ≡⟨ cong (_% suc n) eq ⟩
(v * suc n) % suc n ≡⟨ m*n%n≡0 v n ⟩
0 ∎
where open ≤-Reasoning
m%n≡0⇔n∣m : ∀ m n → m % suc n ≡ 0 ⇔ suc n ∣ m
m%n≡0⇔n∣m m n = equivalence (m%n≡0⇒n∣m m n) (n∣m⇒m%n≡0 m n)
------------------------------------------------------------------------
-- Properties of _∣_ and _≤_
∣⇒≤ : ∀ {m n} → m ∣ suc n → m ≤ suc n
∣⇒≤ {m} {n} (divides (suc q) eq) = begin
m ≤⟨ m≤m+n m (q * m) ⟩
suc q * m ≡⟨ sym eq ⟩
suc n ∎
where open ≤-Reasoning
>⇒∤ : ∀ {m n} → m > suc n → m ∤ suc n
>⇒∤ (s≤s m>n) m∣n = contradiction (∣⇒≤ m∣n) (≤⇒≯ m>n)
------------------------------------------------------------------------
-- _∣_ is a partial order
∣-reflexive : _≡_ ⇒ _∣_
∣-reflexive {n} refl = divides 1 (sym (*-identityˡ n))
∣-refl : Reflexive _∣_
∣-refl = ∣-reflexive refl
∣-trans : Transitive _∣_
∣-trans (divides p refl) (divides q refl) =
divides (q * p) (sym (*-assoc q p _))
∣-antisym : Antisymmetric _≡_ _∣_
∣-antisym {m} {zero} _ (divides q refl) = *-zeroʳ q
∣-antisym {zero} {n} (divides p eq) _ = sym (trans eq (*-comm p 0))
∣-antisym {suc m} {suc n} p∣q q∣p = ≤-antisym (∣⇒≤ p∣q) (∣⇒≤ q∣p)
infix 4 _∣?_
_∣?_ : Decidable _∣_
zero ∣? zero = yes (divides 0 refl)
zero ∣? suc m = no ((λ()) ∘′ ∣-antisym (divides 0 refl))
suc n ∣? m = Dec.map (m%n≡0⇔n∣m m n) (m % suc n ≟ 0)
∣-isPreorder : IsPreorder _≡_ _∣_
∣-isPreorder = record
{ isEquivalence = PropEq.isEquivalence
; reflexive = ∣-reflexive
; trans = ∣-trans
}
∣-isPartialOrder : IsPartialOrder _≡_ _∣_
∣-isPartialOrder = record
{ isPreorder = ∣-isPreorder
; antisym = ∣-antisym
}
∣-preorder : Preorder 0ℓ 0ℓ 0ℓ
∣-preorder = record
{ isPreorder = ∣-isPreorder
}
∣-poset : Poset 0ℓ 0ℓ 0ℓ
∣-poset = record
{ isPartialOrder = ∣-isPartialOrder
}
------------------------------------------------------------------------
-- A reasoning module for the _∣_ relation
module ∣-Reasoning where
private
module Base = PreorderReasoning ∣-preorder
open Base public
hiding (step-≈; step-≈˘; step-∼)
infixr 2 step-∣
step-∣ = Base.step-∼
syntax step-∣ x y∣z x∣y = x ∣⟨ x∣y ⟩ y∣z
------------------------------------------------------------------------
-- Simple properties of _∣_
infix 10 1∣_ _∣0
1∣_ : ∀ n → 1 ∣ n
1∣ n = divides n (sym (*-identityʳ n))
_∣0 : ∀ n → n ∣ 0
n ∣0 = divides 0 refl
0∣⇒≡0 : ∀ {n} → 0 ∣ n → n ≡ 0
0∣⇒≡0 {n} 0∣n = ∣-antisym (n ∣0) 0∣n
∣1⇒≡1 : ∀ {n} → n ∣ 1 → n ≡ 1
∣1⇒≡1 {n} n∣1 = ∣-antisym n∣1 (1∣ n)
n∣n : ∀ {n} → n ∣ n
n∣n {n} = ∣-refl
------------------------------------------------------------------------
-- Properties of _∣_ and _+_
∣m∣n⇒∣m+n : ∀ {i m n} → i ∣ m → i ∣ n → i ∣ m + n
∣m∣n⇒∣m+n (divides p refl) (divides q refl) =
divides (p + q) (sym (*-distribʳ-+ _ p q))
∣m+n∣m⇒∣n : ∀ {i m n} → i ∣ m + n → i ∣ m → i ∣ n
∣m+n∣m⇒∣n {i} {m} {n} (divides p m+n≡p*i) (divides q m≡q*i) =
divides (p ∸ q) $ begin-equality
n ≡⟨ sym (m+n∸n≡m n m) ⟩
n + m ∸ m ≡⟨ cong (_∸ m) (+-comm n m) ⟩
m + n ∸ m ≡⟨ cong₂ _∸_ m+n≡p*i m≡q*i ⟩
p * i ∸ q * i ≡⟨ sym (*-distribʳ-∸ i p q) ⟩
(p ∸ q) * i ∎
where open ∣-Reasoning
------------------------------------------------------------------------
-- Properties of _∣_ and _*_
n∣m*n : ∀ m {n} → n ∣ m * n
n∣m*n m = divides m refl
m∣m*n : ∀ {m} n → m ∣ m * n
m∣m*n n = divides n (*-comm _ n)
∣m⇒∣m*n : ∀ {i m} n → i ∣ m → i ∣ m * n
∣m⇒∣m*n {i} {m} n (divides q refl) = ∣-trans (n∣m*n q) (m∣m*n n)
∣n⇒∣m*n : ∀ {i} m {n} → i ∣ n → i ∣ m * n
∣n⇒∣m*n {i} m {n} i∣n = subst (i ∣_) (*-comm n m) (∣m⇒∣m*n m i∣n)
*-monoʳ-∣ : ∀ {i j} k → i ∣ j → k * i ∣ k * j
*-monoʳ-∣ {i} {j} k (divides q refl) = divides q $ begin-equality
k * (q * i) ≡⟨ sym (*-assoc k q i) ⟩
(k * q) * i ≡⟨ cong (_* i) (*-comm k q) ⟩
(q * k) * i ≡⟨ *-assoc q k i ⟩
q * (k * i) ∎
where open ≤-Reasoning
*-monoˡ-∣ : ∀ {i j} k → i ∣ j → i * k ∣ j * k
*-monoˡ-∣ {i} {j} k rewrite *-comm i k | *-comm j k = *-monoʳ-∣ k
*-cancelˡ-∣ : ∀ {i j} k → suc k * i ∣ suc k * j → i ∣ j
*-cancelˡ-∣ {i} {j} k (divides q eq) =
divides q $ *-cancelʳ-≡ j (q * i) $ begin-equality
j * (suc k) ≡⟨ *-comm j (suc k) ⟩
suc k * j ≡⟨ eq ⟩
q * (suc k * i) ≡⟨ cong (q *_) (*-comm (suc k) i) ⟩
q * (i * suc k) ≡⟨ sym (*-assoc q i (suc k)) ⟩
(q * i) * suc k ∎
where open ≤-Reasoning
*-cancelʳ-∣ : ∀ {i j} k {k≢0 : False (k ≟ 0)} → i * k ∣ j * k → i ∣ j
*-cancelʳ-∣ {i} {j} k@(suc k-1) rewrite *-comm i k | *-comm j k = *-cancelˡ-∣ k-1
------------------------------------------------------------------------
-- Properties of _∣_ and _∸_
∣m∸n∣n⇒∣m : ∀ i {m n} → n ≤ m → i ∣ m ∸ n → i ∣ n → i ∣ m
∣m∸n∣n⇒∣m i {m} {n} n≤m (divides p m∸n≡p*i) (divides q n≡q*o) =
divides (p + q) $ begin-equality
m ≡⟨ sym (m+[n∸m]≡n n≤m) ⟩
n + (m ∸ n) ≡⟨ +-comm n (m ∸ n) ⟩
m ∸ n + n ≡⟨ cong₂ _+_ m∸n≡p*i n≡q*o ⟩
p * i + q * i ≡⟨ sym (*-distribʳ-+ i p q) ⟩
(p + q) * i ∎
where open ≤-Reasoning
------------------------------------------------------------------------
-- Properties of _∣_ and _/_
m/n∣m : ∀ {m n n≢0} → n ∣ m → (m / n) {n≢0} ∣ m
m/n∣m {m} {n} (divides p refl) = begin
p * n / n ≡⟨ m*n/n≡m p n ⟩
p ∣⟨ m∣m*n n ⟩
p * n ∎
where open ∣-Reasoning
m*n∣o⇒m∣o/n : ∀ m n {o n≢0} → m * n ∣ o → m ∣ (o / n) {n≢0}
m*n∣o⇒m∣o/n m n {_} {≢0} (divides p refl) = begin
m ∣⟨ n∣m*n p ⟩
p * m ≡⟨ sym (*-identityʳ (p * m)) ⟩
p * m * 1 ≡⟨ sym (cong (p * m *_) (n/n≡1 n)) ⟩
p * m * (n / n) ≡⟨ sym (*-/-assoc (p * m) {≢0 = ≢0} (n∣n {n})) ⟩
p * m * n / n ≡⟨ cong (λ v → (v / n) {≢0}) (*-assoc p m n) ⟩
p * (m * n) / n ∎
where open ∣-Reasoning
m*n∣o⇒n∣o/m : ∀ m n {o n≢0} → m * n ∣ o → n ∣ (o / m) {n≢0}
m*n∣o⇒n∣o/m m n {o} {≢0} rewrite *-comm m n = m*n∣o⇒m∣o/n n m {o} {≢0}
m∣n/o⇒m*o∣n : ∀ {m n o n≢0} → o ∣ n → m ∣ (n / o) {n≢0} → m * o ∣ n
m∣n/o⇒m*o∣n {m} {n} {o} (divides p refl) m∣p*o/o = begin
m * o ∣⟨ *-monoˡ-∣ o (subst (m ∣_) (m*n/n≡m p o) m∣p*o/o) ⟩
p * o ∎
where open ∣-Reasoning
m∣n/o⇒o*m∣n : ∀ {m n o o≢0} → o ∣ n → m ∣ (n / o) {o≢0} → o * m ∣ n
m∣n/o⇒o*m∣n {m} {_} {o} {≢0} rewrite *-comm o m = m∣n/o⇒m*o∣n {n≢0 = ≢0}
m/n∣o⇒m∣o*n : ∀ {m n o n≢0} → n ∣ m → (m / n) {n≢0} ∣ o → m ∣ o * n
m/n∣o⇒m∣o*n {_} {n} {o} (divides p refl) p*n/n∣o = begin
p * n ∣⟨ *-monoˡ-∣ n (subst (_∣ o) (m*n/n≡m p n) p*n/n∣o) ⟩
o * n ∎
where open ∣-Reasoning
m∣n*o⇒m/n∣o : ∀ {m n o n≢0} → n ∣ m → m ∣ o * n → (m / n) {n≢0} ∣ o
m∣n*o⇒m/n∣o {_} {n@(suc _)} {o} (divides p refl) pn∣on = begin
p * n / n ≡⟨ m*n/n≡m p n ⟩
p ∣⟨ *-cancelʳ-∣ n pn∣on ⟩
o ∎
where open ∣-Reasoning
------------------------------------------------------------------------
-- Properties of _∣_ and _%_
∣n∣m%n⇒∣m : ∀ {m n d ≢0} → d ∣ n → d ∣ (m % n) {≢0} → d ∣ m
∣n∣m%n⇒∣m {m} {n@(suc n-1)} {d} (divides a n≡ad) (divides b m%n≡bd) =
divides (b + (m / n) * a) (begin-equality
m ≡⟨ m≡m%n+[m/n]*n m n-1 ⟩
m % n + (m / n) * n ≡⟨ cong₂ _+_ m%n≡bd (cong (m / n *_) n≡ad) ⟩
b * d + (m / n) * (a * d) ≡⟨ sym (cong (b * d +_) (*-assoc (m / n) a d)) ⟩
b * d + ((m / n) * a) * d ≡⟨ sym (*-distribʳ-+ d b _) ⟩
(b + (m / n) * a) * d ∎)
where open ≤-Reasoning
%-presˡ-∣ : ∀ {m n d ≢0} → d ∣ m → d ∣ n → d ∣ (m % n) {≢0}
%-presˡ-∣ {m} {n@(suc n-1)} {d} (divides a refl) (divides b 1+n≡bd) =
divides (a ∸ ad/n * b) $ begin-equality
a * d % n ≡⟨ m%n≡m∸m/n*n (a * d) n-1 ⟩
a * d ∸ ad/n * n ≡⟨ cong (λ v → a * d ∸ ad/n * v) 1+n≡bd ⟩
a * d ∸ ad/n * (b * d) ≡⟨ sym (cong (a * d ∸_) (*-assoc ad/n b d)) ⟩
a * d ∸ (ad/n * b) * d ≡⟨ sym (*-distribʳ-∸ d a (ad/n * b)) ⟩
(a ∸ ad/n * b) * d ∎
where open ≤-Reasoning; ad/n = a * d / n
------------------------------------------------------------------------
-- DEPRECATED - please use new names as continuing support for the old
-- names is not guaranteed.
-- Version 0.14
∣-+ = ∣m∣n⇒∣m+n
{-# WARNING_ON_USAGE ∣-+
"Warning: ∣-+ was deprecated in v0.14.
Please use ∣m∣n⇒∣m+n instead."
#-}
∣-∸ = ∣m+n∣m⇒∣n
{-# WARNING_ON_USAGE ∣-∸
"Warning: ∣-∸ was deprecated in v0.14.
Please use ∣m+n∣m⇒∣n instead."
#-}
∣-* = n∣m*n
{-# WARNING_ON_USAGE ∣-*
"Warning: ∣-* was deprecated in v0.14.
Please use n∣m*n instead."
#-}
-- Version 0.17
open import Data.Fin.Base using (Fin; zero; suc; toℕ)
import Data.Fin.Properties as FP
open import Data.Nat.Solver
open +-*-Solver
nonZeroDivisor-lemma : ∀ m q (r : Fin (1 + m)) → toℕ r ≢ 0 →
1 + m ∤ toℕ r + q * (1 + m)
nonZeroDivisor-lemma m zero r r≢zero (divides zero eq) = r≢zero $ begin-equality
toℕ r ≡⟨ sym (*-identityˡ (toℕ r)) ⟩
1 * toℕ r ≡⟨ eq ⟩
0 ∎
where open ≤-Reasoning
nonZeroDivisor-lemma m zero r r≢zero (divides (suc q) eq) =
m+1+n≰m m $ begin
m + suc (q * suc m) ≡⟨ +-suc m (q * suc m) ⟩
suc (m + q * suc m) ≡⟨ sym eq ⟩
1 * toℕ r ≡⟨ *-identityˡ (toℕ r) ⟩
toℕ r ≤⟨ FP.toℕ≤pred[n] r ⟩
m ∎
where open ≤-Reasoning
nonZeroDivisor-lemma m (suc q) r r≢zero d =
nonZeroDivisor-lemma m q r r≢zero (∣m+n∣m⇒∣n d' ∣-refl)
where
lem = solve 3 (λ m r q → r :+ (m :+ q) := m :+ (r :+ q))
refl (suc m) (toℕ r) (q * suc m)
d' = subst (1 + m ∣_) lem d
{-# WARNING_ON_USAGE nonZeroDivisor-lemma
"Warning: nonZeroDivisor-lemma was deprecated in v0.17."
#-}
-- Version 1.1
poset = ∣-poset
{-# WARNING_ON_USAGE poset
"Warning: poset was deprecated in v1.1.
Please use ∣-poset instead."
#-}
*-cong = *-monoʳ-∣
{-# WARNING_ON_USAGE *-cong
"Warning: *-cong was deprecated in v1.1.
Please use *-monoʳ-∣ instead."
#-}
/-cong = *-cancelˡ-∣
{-# WARNING_ON_USAGE /-cong
"Warning: /-cong was deprecated in v1.1.
Please use *-cancelˡ-∣ instead."
#-}
| {
"alphanum_fraction": 0.450563976,
"avg_line_length": 31.9661971831,
"ext": "agda",
"hexsha": "888d88463f2615d4c1d4605d12b46130d68e0386",
"lang": "Agda",
"max_forks_count": 1,
"max_forks_repo_forks_event_max_datetime": "2021-11-04T06:54:45.000Z",
"max_forks_repo_forks_event_min_datetime": "2021-11-04T06:54:45.000Z",
"max_forks_repo_head_hexsha": "fb380f2e67dcb4a94f353dbaec91624fcb5b8933",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "DreamLinuxer/popl21-artifact",
"max_forks_repo_path": "agda-stdlib/src/Data/Nat/Divisibility.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "fb380f2e67dcb4a94f353dbaec91624fcb5b8933",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "DreamLinuxer/popl21-artifact",
"max_issues_repo_path": "agda-stdlib/src/Data/Nat/Divisibility.agda",
"max_line_length": 81,
"max_stars_count": 5,
"max_stars_repo_head_hexsha": "fb380f2e67dcb4a94f353dbaec91624fcb5b8933",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "DreamLinuxer/popl21-artifact",
"max_stars_repo_path": "agda-stdlib/src/Data/Nat/Divisibility.agda",
"max_stars_repo_stars_event_max_datetime": "2020-10-10T21:41:32.000Z",
"max_stars_repo_stars_event_min_datetime": "2020-10-07T12:07:53.000Z",
"num_tokens": 5401,
"size": 11348
} |
import Relation.Unary.Monotone as Mono
open import Data.List.Prefix
open import Data.List as List
module Category.Monad.Monotone.Heap.HList
(T : Set)
(V : T → List T → Set)⦃ wkV : ∀ {a} → Mono.Monotone ⊑-preorder (V a) ⦄ where
open import Level
open import Data.List.All as All
open import Data.List.All.Properties.Extra
open import Data.List.Any
open import Data.List.Membership.Propositional using (_∈_)
open import Data.List.Properties.Extra
open import Data.Product
open import Data.Unit
open import Relation.Binary using (Preorder)
open import Relation.Unary hiding (_∈_)
open import Relation.Unary.PredicateTransformer using (Pt)
open import Relation.Unary.Monotone.Prefix {T = T}
private
HeapT : Set
HeapT = List T
Heap : Pred HeapT _
Heap = λ W → All (λ a → V a W) W
open Mono (⊑-preorder {A = T})
open import Category.Monad.Monotone (⊑-preorder {A = T})
open import Category.Monad.Monotone.State ⊑-preorder Heap
open import Category.Monad.Monotone.Heap ⊑-preorder T V Heap _∈_
open import Category.Monad using (RawMonad)
module _ {M : Set → Set}⦃ Mon : RawMonad M ⦄ where
private module M = RawMonad Mon
hlist-heap-monad : HeapMonad (MST M)
HeapMonad.store hlist-heap-monad {a}{i} sv μ =
let ext = ∷ʳ-⊒ a i in M.return (_ , ext , (wk ext μ all-∷ʳ wk ext sv) , ∈-∷ʳ i a )
HeapMonad.modify hlist-heap-monad ptr v μ =
M.return (_ , ⊑-refl , μ All[ ptr ]≔' v , lift tt)
HeapMonad.deref hlist-heap-monad ptr μ =
M.return (_ , ⊑-refl , μ , ∈-all ptr μ)
| {
"alphanum_fraction": 0.703802535,
"avg_line_length": 31.8936170213,
"ext": "agda",
"hexsha": "96d8bd1c779ad239adea827192fa7471aeed591e",
"lang": "Agda",
"max_forks_count": 1,
"max_forks_repo_forks_event_max_datetime": "2021-12-28T17:38:05.000Z",
"max_forks_repo_forks_event_min_datetime": "2021-12-28T17:38:05.000Z",
"max_forks_repo_head_hexsha": "0c096fea1716d714db0ff204ef2a9450b7a816df",
"max_forks_repo_licenses": [
"Apache-2.0"
],
"max_forks_repo_name": "metaborg/mj.agda",
"max_forks_repo_path": "src/Category/Monad/Monotone/Heap/HList.agda",
"max_issues_count": 1,
"max_issues_repo_head_hexsha": "0c096fea1716d714db0ff204ef2a9450b7a816df",
"max_issues_repo_issues_event_max_datetime": "2020-10-14T13:41:58.000Z",
"max_issues_repo_issues_event_min_datetime": "2019-01-13T13:03:47.000Z",
"max_issues_repo_licenses": [
"Apache-2.0"
],
"max_issues_repo_name": "metaborg/mj.agda",
"max_issues_repo_path": "src/Category/Monad/Monotone/Heap/HList.agda",
"max_line_length": 86,
"max_stars_count": 10,
"max_stars_repo_head_hexsha": "0c096fea1716d714db0ff204ef2a9450b7a816df",
"max_stars_repo_licenses": [
"Apache-2.0"
],
"max_stars_repo_name": "metaborg/mj.agda",
"max_stars_repo_path": "src/Category/Monad/Monotone/Heap/HList.agda",
"max_stars_repo_stars_event_max_datetime": "2021-09-24T08:02:33.000Z",
"max_stars_repo_stars_event_min_datetime": "2017-11-17T17:10:36.000Z",
"num_tokens": 482,
"size": 1499
} |
import Relation.Binary.PropositionalEquality
module Data.Bin.Multiplication where
private module PropEq = Relation.Binary.PropositionalEquality
module ℕ-lemmas where
open import Data.Nat
open import Data.Nat.Properties
open import Relation.Binary.PropositionalEquality
open SemiringSolver
*-2-3-comm : ∀ x y z → x * y * z ≡ x * z * y
*-2-3-comm x y z = solve 3 (λ x y z → x :* y :* z := x :* z :* y) refl x y z
n+x≡0→n≡0 : ∀ {n x} → n + x ≡ 0 → n ≡ 0
n+x≡0→n≡0 {zero} = λ _ → refl
n+x≡0→n≡0 {suc _} = λ ()
distribʳ : ∀ a b c → (a + b) * c ≡ a * c + b * c
distribʳ a b c = solve 3 (λ a b c → (a :+ b) :* c := a :* c :+ b :* c) refl a b c
open PropEq using (_≡_; cong; cong₂; trans; sym; [_]; inspect)
open import Data.Bin using (_*2; toℕ; 0#; _1#; Bin; pred; _*_; _+_)
open import Data.Nat using (ℕ; zero; suc)
renaming (_*_ to _ℕ*_; _+_ to _ℕ+_)
open import Data.Nat.Properties using (isCommutativeSemiring)
open import Algebra.Structures
using (module IsCommutativeSemiring;
module IsCommutativeMonoid)
open IsCommutativeSemiring isCommutativeSemiring
using (+-isCommutativeMonoid; *-isCommutativeMonoid)
open import Data.Product
open import Relation.Nullary
open import Data.Fin using (zero; suc) renaming (toℕ to bitToℕ)
open import Data.Digit using (Bit)
open import Data.List using (List; _∷_; [])
open import Data.Bin.Utils
open import Data.Bin.Bijection using (fromℕ-bijection; toℕ-inj)
import Relation.Binary.PropositionalEquality
open Relation.Binary.PropositionalEquality.≡-Reasoning
import Data.Bin.Addition
open Data.Bin.Addition using (+-is-addition)
module B+ICM = IsCommutativeMonoid Data.Bin.Addition.is-commutativeMonoid
open B+ICM using () renaming (identity to +-identity; ∙-cong to +-cong)
*2-is-*2 : ∀ x → toℕ (x *2) ≡ toℕ x ℕ* 2
*2-is-*2 0# = PropEq.refl
*2-is-*2 (bs 1#) = PropEq.refl
bitToX-≡ : ∀ x → bitToℕ x ≡ toℕ (bitToBin x)
bitToX-≡ zero = PropEq.refl
bitToX-≡ (suc zero) = PropEq.refl
bitToX-≡ (suc (suc ()))
∷1#-interpretation : ∀ (b : Bit) (bs : List Bit) → ((b ∷ bs) 1#) ≡ bitToBin b + (bs 1#) *2
∷1#-interpretation b bs = toℕ-inj (
begin
toℕ ((b ∷ bs) 1#)
≡⟨ PropEq.refl ⟩
bitToℕ b ℕ+ toℕ (bs 1#) ℕ* 2
≡⟨ cong₂ _ℕ+_ (bitToX-≡ b) (sym (*2-is-*2 (bs 1#))) ⟩
toℕ (bitToBin b) ℕ+ toℕ ((bs 1#) *2)
≡⟨ sym (+-is-addition (bitToBin b) ((bs 1#) *2)) ⟩
toℕ (bitToBin b + (bs 1#) *2)
∎)
open import Function using (_⟨_⟩_)
multBit : Bit → Bin → Bin
multBit zero _ = 0#
multBit (suc zero) n = n
multBit (suc (suc ())) _
n+x≡0→n≡0 : ∀ {n x} → n + x ≡ 0# → n ≡ 0#
n+x≡0→n≡0 {n} {x} n+x≡0 = toℕ-inj (ℕ-lemmas.n+x≡0→n≡0 ((sym (+-is-addition n x)) ⟨ trans ⟩ cong toℕ n+x≡0))
1+*n≡0→n≡0 : ∀ {l} n → l 1# * n ≡ 0# → n ≡ 0#
1+*n≡0→n≡0 {[]} n eq = eq
1+*n≡0→n≡0 {h ∷ t} n eq with t 1# * n | PropEq.inspect (λ n → (t 1# * n)) n
1+*n≡0→n≡0 {h ∷ t} n _ | 0# | [ eq ] = 1+*n≡0→n≡0 {t} n eq
1+*n≡0→n≡0 {zero ∷ t} n eq | (l 1#) | [ eq2 ] rewrite eq2 with eq
... | ()
1+*n≡0→n≡0 {suc zero ∷ t} n eq | (l 1#) | [ eq2 ] rewrite eq2 = n+x≡0→n≡0 {n} {(zero ∷ l) 1#} eq
1+*n≡0→n≡0 {suc (suc ()) ∷ t} n eq | _ | _
simplify-mult : ∀ x xs n → (x ∷ xs) 1# * n ≡ multBit x n + (xs 1# * n) *2
simplify-mult x xs n with (xs 1# * n) | inspect (λ n → (xs 1# * n)) n
simplify-mult zero xs n | 0# | [ ≡ ] rewrite ≡ = PropEq.refl
simplify-mult (suc zero) xs n | 0# | [ ≡ ] rewrite ≡ | 1+*n≡0→n≡0 {xs} n ≡ = PropEq.refl
simplify-mult zero xs n | (xs' 1#) | [ ≡ ] rewrite ≡ =
begin
(zero ∷ xs') 1#
≡⟨ PropEq.refl ⟩
(xs' 1#) *2
≡⟨ B+ICM.sym ( B+ICM.identityˡ ((xs' 1#) *2)) ⟩
0# + (xs' 1#) *2
≡⟨ PropEq.refl ⟩
multBit zero n + (xs' 1#) *2
∎
simplify-mult (suc zero) xs n | (xs' 1#) | [ ≡ ] rewrite ≡ =
begin
n + (zero ∷ xs') 1#
≡⟨ PropEq.refl ⟩
multBit (suc zero) n + (xs' 1#) *2
∎
simplify-mult (suc (suc ())) xs n | _ | _
_*-def'_ : ℕ → Bin → Bin
zero *-def' y = 0#
(suc x) *-def' y = y + (x *-def' y)
_*-def_ : Bin → Bin → Bin
x *-def y = (toℕ x) *-def' y
infixl 7 _*-def_
*-def'-is-* : ∀ m n → toℕ (m *-def' n) ≡ m ℕ* toℕ n
*-def'-is-* zero n = PropEq.refl
*-def'-is-* (suc m) n = +-is-addition n ( m *-def' n) ⟨ trans ⟩ cong (_ℕ+_ (toℕ n)) (*-def'-is-* m n)
*-def-is-* : ∀ m n → toℕ (m *-def n) ≡ toℕ m ℕ* toℕ n
*-def-is-* m = *-def'-is-* (toℕ m)
*-def-*2-comm : ∀ x y → (x *-def y) *2 ≡ x *2 *-def y
*-def-*2-comm x y = toℕ-inj (
begin
toℕ ((x *-def y) *2)
≡⟨ *2-is-*2 (x *-def y) ⟩
toℕ (x *-def y) ℕ* 2
≡⟨ cong (λ x → x ℕ* 2) (*-def-is-* x y) ⟩
toℕ x ℕ* toℕ y ℕ* 2
≡⟨ ℕ-lemmas.*-2-3-comm (toℕ x) (toℕ y) 2 ⟩
toℕ x ℕ* 2 ℕ* toℕ y
≡⟨ cong (λ x → x ℕ* toℕ y) (sym (*2-is-*2 x)) ⟩
toℕ (x *2) ℕ* toℕ y
≡⟨ sym (*-def-is-* (x *2) y) ⟩
toℕ (x *2 *-def y)
∎)
multbit-is-*-def : ∀ c x → multBit c x ≡ bitToBin c *-def x
multbit-is-*-def zero x = PropEq.refl
multbit-is-*-def (suc zero) x = sym (proj₂ +-identity x)
multbit-is-*-def (suc (suc ())) x
*-def-distribʳ : ∀ a b c → (a + b) *-def c ≡ a *-def c + b *-def c
*-def-distribʳ a b c = toℕ-inj (
begin
toℕ ((a + b) *-def c)
≡⟨ *-def-is-* (a + b) c ⟩
toℕ (a + b) ℕ* toℕ c
≡⟨ cong (λ x → x ℕ* toℕ c) (+-is-addition a b) ⟩
(toℕ a ℕ+ toℕ b) ℕ* toℕ c
≡⟨ ℕ-lemmas.distribʳ (toℕ a) (toℕ b) (toℕ c) ⟩
toℕ a ℕ* toℕ c ℕ+ toℕ b ℕ* toℕ c
≡⟨ cong₂ _ℕ+_ (kojo a) (kojo b) ⟩
toℕ (a *-def c) ℕ+ toℕ (b *-def c)
≡⟨ sym (+-is-addition (a *-def c) (b *-def c)) ⟩
toℕ (a *-def c + b *-def c)
∎
) where
kojo : ∀ x → toℕ x ℕ* toℕ c ≡ toℕ (x *-def c)
kojo x = sym (*-def-is-* x c)
mutual
*-is-*-def : ∀ m n → m * n ≡ m *-def n
*-is-*-def 0# n = PropEq.refl
*-is-*-def (l 1#) n = *-is-*-def-1# l n
*-is-*-def-1# : ∀ l n → l 1# * n ≡ l 1# *-def n
*-is-*-def-1# [] n = sym (proj₂ +-identity n)
*-is-*-def-1# (x ∷ xs) n = *-is-*-def-∷ x xs n
*-is-*-def-∷ : ∀ h t n → (h ∷ t) 1# * n ≡ ((h ∷ t) 1#) *-def n
*-is-*-def-∷ h t n =
begin
(h ∷ t) 1# * n
≡⟨ simplify-mult h t n ⟩
multBit h n + (t 1# * n) *2
≡⟨ +-cong (multbit-is-*-def h n) (cong (λ x → x *2) (*-is-*-def-1# t n) ⟨ trans ⟩ *-def-*2-comm (t 1#) n) ⟩
bitToBin h *-def n + t 1# *2 *-def n
≡⟨ sym (*-def-distribʳ (bitToBin h) (t 1# *2) n) ⟩
(bitToBin h + t 1# *2) *-def n
≡⟨ cong (λ x → x *-def n) (sym (∷1#-interpretation h t)) ⟩
((h ∷ t) 1#) *-def n
∎
*-*2-comm : ∀ x y → (x * y) *2 ≡ x *2 * y
*-*2-comm x y = cong _*2 (*-is-*-def x y) ⟨ trans ⟩ *-def-*2-comm x y ⟨ trans ⟩ sym (*-is-*-def (x *2) y)
*-distribʳ : ∀ a b c → (a + b) * c ≡ a * c + b * c
*-distribʳ a b c =
*-is-*-def (a + b) c
⟨ trans ⟩ *-def-distribʳ a b c
⟨ trans ⟩ sym (cong₂ _+_ (*-is-*-def a c) (*-is-*-def b c))
*-is-multiplication : ∀ a b → toℕ (a * b) ≡ toℕ a ℕ* toℕ b
*-is-multiplication a b = cong toℕ (*-is-*-def a b) ⟨ trans ⟩ *-def-is-* a b
| {
"alphanum_fraction": 0.4984696717,
"avg_line_length": 34.8932038835,
"ext": "agda",
"hexsha": "ea26434109531dd5636b56bcf2993f654fdecf06",
"lang": "Agda",
"max_forks_count": null,
"max_forks_repo_forks_event_max_datetime": null,
"max_forks_repo_forks_event_min_datetime": null,
"max_forks_repo_head_hexsha": "09cc5104421e88da82f9fead5a43f0028f77810d",
"max_forks_repo_licenses": [
"Unlicense"
],
"max_forks_repo_name": "Rotsor/BinDivMod",
"max_forks_repo_path": "Data/Bin/Multiplication.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "09cc5104421e88da82f9fead5a43f0028f77810d",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"Unlicense"
],
"max_issues_repo_name": "Rotsor/BinDivMod",
"max_issues_repo_path": "Data/Bin/Multiplication.agda",
"max_line_length": 114,
"max_stars_count": 1,
"max_stars_repo_head_hexsha": "09cc5104421e88da82f9fead5a43f0028f77810d",
"max_stars_repo_licenses": [
"Unlicense"
],
"max_stars_repo_name": "Rotsor/BinDivMod",
"max_stars_repo_path": "Data/Bin/Multiplication.agda",
"max_stars_repo_stars_event_max_datetime": "2019-11-18T13:58:14.000Z",
"max_stars_repo_stars_event_min_datetime": "2019-11-18T13:58:14.000Z",
"num_tokens": 3448,
"size": 7188
} |
{-# OPTIONS --without-K #-}
module Base where
open import Types public
open import Functions public
open import Paths public
open import HLevel public
open import Equivalences public
open import Univalence public
open import Funext public
open import EquivalenceLemmas public
open import HLevelBis public
open import FiberEquivalences public
| {
"alphanum_fraction": 0.8313953488,
"avg_line_length": 22.9333333333,
"ext": "agda",
"hexsha": "caa686cc25f60828bc70c12c45669e7c66c51b48",
"lang": "Agda",
"max_forks_count": 50,
"max_forks_repo_forks_event_max_datetime": "2022-02-14T03:03:25.000Z",
"max_forks_repo_forks_event_min_datetime": "2015-01-10T01:48:08.000Z",
"max_forks_repo_head_hexsha": "939a2d83e090fcc924f69f7dfa5b65b3b79fe633",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "nicolaikraus/HoTT-Agda",
"max_forks_repo_path": "old/Base.agda",
"max_issues_count": 31,
"max_issues_repo_head_hexsha": "939a2d83e090fcc924f69f7dfa5b65b3b79fe633",
"max_issues_repo_issues_event_max_datetime": "2021-10-03T19:15:25.000Z",
"max_issues_repo_issues_event_min_datetime": "2015-03-05T20:09:00.000Z",
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "nicolaikraus/HoTT-Agda",
"max_issues_repo_path": "old/Base.agda",
"max_line_length": 36,
"max_stars_count": 294,
"max_stars_repo_head_hexsha": "f8fa68bf753d64d7f45556ca09d0da7976709afa",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "UlrikBuchholtz/HoTT-Agda",
"max_stars_repo_path": "old/Base.agda",
"max_stars_repo_stars_event_max_datetime": "2022-03-20T13:54:45.000Z",
"max_stars_repo_stars_event_min_datetime": "2015-01-09T16:23:23.000Z",
"num_tokens": 75,
"size": 344
} |
-- Andreas, 2013-11-07
-- Need to drop parameters not only from constructors found by
-- instance search, but also from projection(like) functions.
module Issue670b where
open import Common.Prelude
open import Common.Equality
record Wrap (A : Set) : Set where
constructor wrap
field
unwrap : A
open Wrap
module _ {A : Set} where
g : {{i : Wrap A → A}} → Wrap A → A
g {{i}} = i
test : g (wrap true) ≡ true
test = refl
-- Error WAS:
-- unwrap Bool (wrap true) != true of type Bool
-- when checking that the expression refl has type
-- g (wrap true) ≡ true
-- Should work now.
| {
"alphanum_fraction": 0.676222597,
"avg_line_length": 20.4482758621,
"ext": "agda",
"hexsha": "6e3e41eccd0130aaa4c61a428eba3e4665986645",
"lang": "Agda",
"max_forks_count": 1,
"max_forks_repo_forks_event_max_datetime": "2022-03-12T11:35:18.000Z",
"max_forks_repo_forks_event_min_datetime": "2022-03-12T11:35:18.000Z",
"max_forks_repo_head_hexsha": "70c8a575c46f6a568c7518150a1a64fcd03aa437",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "masondesu/agda",
"max_forks_repo_path": "test/succeed/Issue670b.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "70c8a575c46f6a568c7518150a1a64fcd03aa437",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "masondesu/agda",
"max_issues_repo_path": "test/succeed/Issue670b.agda",
"max_line_length": 62,
"max_stars_count": 1,
"max_stars_repo_head_hexsha": "477c8c37f948e6038b773409358fd8f38395f827",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "larrytheliquid/agda",
"max_stars_repo_path": "test/succeed/Issue670b.agda",
"max_stars_repo_stars_event_max_datetime": "2018-10-10T17:08:44.000Z",
"max_stars_repo_stars_event_min_datetime": "2018-10-10T17:08:44.000Z",
"num_tokens": 171,
"size": 593
} |
------------------------------------------------------------------------------
-- Alter: An unguarded co-recursive function
------------------------------------------------------------------------------
{-# OPTIONS --exact-split #-}
{-# OPTIONS --no-sized-types #-}
{-# OPTIONS --no-universe-polymorphism #-}
{-# OPTIONS --without-K #-}
module FOT.FOTC.UnguardedCorecursion.Alter.Alter where
open import FOTC.Base
open import FOTC.Base.List
open import FOTC.Data.Bool
open import FOTC.Data.List
------------------------------------------------------------------------------
postulate
alter : D
alter-eq : alter ≡ true ∷ false ∷ alter
{-# ATP axiom alter-eq #-}
postulate
not₀ : D
not₀-eq : ∀ b → not₀ · b ≡ not b
{-# ATP axiom not₀-eq #-}
postulate
alter' : D
alter'-eq : alter' ≡ true ∷ map not₀ alter'
{-# ATP axiom alter'-eq #-}
| {
"alphanum_fraction": 0.4525139665,
"avg_line_length": 27.1212121212,
"ext": "agda",
"hexsha": "de90d74642331f673e79b82c5d3e145fe900b178",
"lang": "Agda",
"max_forks_count": 3,
"max_forks_repo_forks_event_max_datetime": "2018-03-14T08:50:00.000Z",
"max_forks_repo_forks_event_min_datetime": "2016-09-19T14:18:30.000Z",
"max_forks_repo_head_hexsha": "2fc9f2b81052a2e0822669f02036c5750371b72d",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "asr/fotc",
"max_forks_repo_path": "notes/FOT/FOTC/UnguardedCorecursion/Alter/Alter.agda",
"max_issues_count": 2,
"max_issues_repo_head_hexsha": "2fc9f2b81052a2e0822669f02036c5750371b72d",
"max_issues_repo_issues_event_max_datetime": "2017-01-01T14:34:26.000Z",
"max_issues_repo_issues_event_min_datetime": "2016-10-12T17:28:16.000Z",
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "asr/fotc",
"max_issues_repo_path": "notes/FOT/FOTC/UnguardedCorecursion/Alter/Alter.agda",
"max_line_length": 78,
"max_stars_count": 11,
"max_stars_repo_head_hexsha": "2fc9f2b81052a2e0822669f02036c5750371b72d",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "asr/fotc",
"max_stars_repo_path": "notes/FOT/FOTC/UnguardedCorecursion/Alter/Alter.agda",
"max_stars_repo_stars_event_max_datetime": "2021-09-12T16:09:54.000Z",
"max_stars_repo_stars_event_min_datetime": "2015-09-03T20:53:42.000Z",
"num_tokens": 198,
"size": 895
} |
{-# OPTIONS --allow-unsolved-metas #-}
-- Andreas, 2014-11-25, issue found by Christopher Jenkins
-- {-# OPTIONS -v tc.with:40 #-}
open import Common.Prelude
open import Common.Equality
infixr 5 _∷_
data Vec (A : Set) : Nat → Set where
[] : Vec A zero
_∷_ : {n : Nat} (x : A) (xs : Vec A n) → Vec A (suc n)
+-suc : ∀ (n m : Nat) → n + suc m ≡ suc (n + m)
+-suc zero m = refl
+-suc (suc n) m = cong suc (+-suc n m)
swap : ∀ {A : Set} n → Vec A (n + n) → Vec A (n + n)
swap zero [] = []
swap (suc n) (x ∷ xs) with n + suc n | +-suc n n
swap (suc n) (x ∷ y ∷ xs) | .(suc (n + n)) | refl = y ∷ x ∷ swap n xs
swap-involutive : ∀ {A : Set} n → (xs : Vec A (n + n)) →
swap n (swap n xs) ≡ xs
swap-involutive zero [] = refl
swap-involutive {A = A} (suc n) (x ∷ xs) with swap {A = A} (suc n)
... | f = {!!}
-- Goal before with is:
-- swap (suc n) (swap (suc n) (x ∷ xs) | n + suc n | +-suc n n) ≡ x ∷ xs
{- ERROR WAS:
A !=< ℕ of type Set
when checking that the type
{A : Set}
(n : ℕ)
(w : Vec A (suc (n + suc n)) → Vec A (suc (n + suc n)))
(x : A)
(xs : Vec A (n + suc n)) →
w (swap (suc x) (xs ∷ w) | x + suc x | +-suc x x) ≡ x ∷ xs
of the generated with function is well-formed
-}
| {
"alphanum_fraction": 0.5190397351,
"avg_line_length": 28.0930232558,
"ext": "agda",
"hexsha": "78ccb058eb1f5c6bc05663f4df82c4f46c61eb81",
"lang": "Agda",
"max_forks_count": 371,
"max_forks_repo_forks_event_max_datetime": "2022-03-30T19:00:30.000Z",
"max_forks_repo_forks_event_min_datetime": "2015-01-03T14:04:08.000Z",
"max_forks_repo_head_hexsha": "7f58030124fa99dfbf8db376659416f3ad8384de",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "cruhland/agda",
"max_forks_repo_path": "test/Succeed/Issue1369.agda",
"max_issues_count": 4066,
"max_issues_repo_head_hexsha": "7f58030124fa99dfbf8db376659416f3ad8384de",
"max_issues_repo_issues_event_max_datetime": "2022-03-31T21:14:49.000Z",
"max_issues_repo_issues_event_min_datetime": "2015-01-10T11:24:51.000Z",
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "cruhland/agda",
"max_issues_repo_path": "test/Succeed/Issue1369.agda",
"max_line_length": 72,
"max_stars_count": 1989,
"max_stars_repo_head_hexsha": "7f58030124fa99dfbf8db376659416f3ad8384de",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "cruhland/agda",
"max_stars_repo_path": "test/Succeed/Issue1369.agda",
"max_stars_repo_stars_event_max_datetime": "2022-03-30T18:20:48.000Z",
"max_stars_repo_stars_event_min_datetime": "2015-01-09T23:51:16.000Z",
"num_tokens": 496,
"size": 1208
} |
{-
Basic properties about Σ-types
- Characterization of equality in Σ-types using transport ([pathSigma≡sigmaPath])
-}
{-# OPTIONS --cubical --safe #-}
module Cubical.Data.Sigma.Properties where
open import Cubical.Data.Sigma.Base
open import Cubical.Core.Everything
open import Cubical.Foundations.Prelude
open import Cubical.Foundations.Isomorphism
open import Cubical.Foundations.Equiv
open import Cubical.Foundations.Univalence
open import Cubical.Foundations.CartesianKanOps
open import Cubical.Relation.Nullary
open import Cubical.Relation.Nullary.DecidableEq
open import Cubical.Data.Nat.Base
private
variable
ℓ : Level
A : Type ℓ
B : (a : A) → Type ℓ
ΣPathP : ∀ {x y}
→ Σ (fst x ≡ fst y) (λ a≡ → PathP (λ i → B (a≡ i)) (snd x) (snd y))
→ x ≡ y
ΣPathP eq = λ i → (fst eq i) , (snd eq i)
Σ≡ : {x y : Σ A B} →
Σ (fst x ≡ fst y) (λ a≡ → PathP (λ i → B (a≡ i)) (snd x) (snd y)) ≃
(x ≡ y)
Σ≡ {A = A} {B = B} {x} {y} = isoToEquiv (iso intro elim intro-elim elim-intro)
where
intro = ΣPathP
elim : x ≡ y → Σ (fst x ≡ fst y) (λ a≡ → PathP (λ i → B (a≡ i)) (snd x) (snd y ))
elim eq = (λ i → fst (eq i)) , λ i → snd (eq i)
intro-elim : ∀ eq → intro (elim eq) ≡ eq
intro-elim eq = refl
elim-intro : ∀ eq → elim (intro eq) ≡ eq
elim-intro eq = refl
-- Alternative version for path in Σ-types, as in the HoTT book
sigmaPathTransport : (a b : Σ A B) → Type _
sigmaPathTransport {B = B} a b =
Σ (fst a ≡ fst b) (λ p → transport (λ i → B (p i)) (snd a) ≡ snd b)
_Σ≡T_ : (a b : Σ A B) → Type _
a Σ≡T b = sigmaPathTransport a b
-- now we prove that the alternative path space a Σ≡ b is equal to the usual path space a ≡ b
-- forward direction
private
pathSigma-π1 : {a b : Σ A B} → a ≡ b → fst a ≡ fst b
pathSigma-π1 p i = fst (p i)
filler-π2 : {a b : Σ A B} → (p : a ≡ b) → I → (i : I) → B (fst (p i))
filler-π2 {B = B} {a = a} p i =
fill (λ i → B (fst (p i)))
(λ t → λ { (i = i0) → coe0→i (λ j → B (fst (p j))) t (snd a)
; (i = i1) → snd (p t) })
(inS (snd a))
pathSigma-π2 : {a b : Σ A B} → (p : a ≡ b) →
subst B (pathSigma-π1 p) (snd a) ≡ snd b
pathSigma-π2 p i = filler-π2 p i i1
pathSigma→sigmaPath : (a b : Σ A B) → a ≡ b → a Σ≡T b
pathSigma→sigmaPath _ _ p = (pathSigma-π1 p , pathSigma-π2 p)
-- backward direction
private
filler-comp : (a b : Σ A B) → a Σ≡T b → I → I → Σ A B
filler-comp {B = B} a b (p , q) i =
hfill (λ t → λ { (i = i0) → a
; (i = i1) → (p i1 , q t) })
(inS (p i , coe0→i (λ j → B (p j)) i (snd a)))
sigmaPath→pathSigma : (a b : Σ A B) → a Σ≡T b → (a ≡ b)
sigmaPath→pathSigma a b x i = filler-comp a b x i i1
-- first homotopy
private
homotopy-π1 : (a b : Σ A B) →
∀ (x : a Σ≡T b) → pathSigma-π1 (sigmaPath→pathSigma a b x) ≡ fst x
homotopy-π1 a b x i j = fst (filler-comp a b x j (~ i))
homotopy-π2 : (a b : Σ A B) → (p : a Σ≡T b) → (i : I) →
(transport (λ j → B (fst (filler-comp a b p j i))) (snd a) ≡ snd b)
homotopy-π2 {B = B} a b p i j =
comp (λ t → B (fst (filler-comp a b p t (i ∨ j))))
(λ t → λ { (j = i0) → coe0→i (λ t → B (fst (filler-comp a b p t i)))
t (snd a)
; (j = i1) → snd (sigmaPath→pathSigma a b p t)
; (i = i0) → snd (filler-comp a b p t j)
; (i = i1) → filler-π2 (sigmaPath→pathSigma a b p) j t })
(snd a)
pathSigma→sigmaPath→pathSigma : {a b : Σ A B} →
∀ (x : a Σ≡T b) → pathSigma→sigmaPath _ _ (sigmaPath→pathSigma a b x) ≡ x
pathSigma→sigmaPath→pathSigma {a = a} p i =
(homotopy-π1 a _ p i , homotopy-π2 a _ p (~ i))
-- second homotopy
sigmaPath→pathSigma→sigmaPath : {a b : Σ A B} →
∀ (x : a ≡ b) → sigmaPath→pathSigma a b (pathSigma→sigmaPath _ _ x) ≡ x
sigmaPath→pathSigma→sigmaPath {B = B} {a = a} {b = b} p i j =
hcomp (λ t → λ { (i = i1) → (fst (p j) , filler-π2 p t j)
; (i = i0) → filler-comp a b (pathSigma→sigmaPath _ _ p) j t
; (j = i0) → (fst a , snd a)
; (j = i1) → (fst b , filler-π2 p t i1) })
(fst (p j) , coe0→i (λ k → B (fst (p k))) j (snd a))
pathSigma≡sigmaPath : (a b : Σ A B) → (a ≡ b) ≡ (a Σ≡T b)
pathSigma≡sigmaPath a b =
isoToPath (iso (pathSigma→sigmaPath a b)
(sigmaPath→pathSigma a b)
(pathSigma→sigmaPath→pathSigma {a = a})
sigmaPath→pathSigma→sigmaPath)
discreteΣ : Discrete A → ((a : A) → Discrete (B a)) → Discrete (Σ A B)
discreteΣ {B = B} Adis Bdis (a0 , b0) (a1 , b1) = discreteΣ' (Adis a0 a1)
where
discreteΣ' : Dec (a0 ≡ a1) → Dec ((a0 , b0) ≡ (a1 , b1))
discreteΣ' (yes p) = J (λ a1 p → ∀ b1 → Dec ((a0 , b0) ≡ (a1 , b1))) (discreteΣ'') p b1
where
discreteΣ'' : (b1 : B a0) → Dec ((a0 , b0) ≡ (a0 , b1))
discreteΣ'' b1 with Bdis a0 b0 b1
... | (yes q) = yes (transport (ua Σ≡) (refl , q))
... | (no ¬q) = no (λ r → ¬q (subst (λ X → PathP (λ i → B (X i)) b0 b1) (Discrete→isSet Adis a0 a0 (cong fst r) refl) (cong snd r)))
discreteΣ' (no ¬p) = no (λ r → ¬p (cong fst r))
| {
"alphanum_fraction": 0.5340842882,
"avg_line_length": 34.7905405405,
"ext": "agda",
"hexsha": "67e95dffdaa4e3fd11d687be9920c824e2ea1576",
"lang": "Agda",
"max_forks_count": null,
"max_forks_repo_forks_event_max_datetime": null,
"max_forks_repo_forks_event_min_datetime": null,
"max_forks_repo_head_hexsha": "a01973ef7264f9454a40697313a2073c51a6b77a",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "oisdk/cubical",
"max_forks_repo_path": "Cubical/Data/Sigma/Properties.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "a01973ef7264f9454a40697313a2073c51a6b77a",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "oisdk/cubical",
"max_issues_repo_path": "Cubical/Data/Sigma/Properties.agda",
"max_line_length": 140,
"max_stars_count": null,
"max_stars_repo_head_hexsha": "a01973ef7264f9454a40697313a2073c51a6b77a",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "oisdk/cubical",
"max_stars_repo_path": "Cubical/Data/Sigma/Properties.agda",
"max_stars_repo_stars_event_max_datetime": null,
"max_stars_repo_stars_event_min_datetime": null,
"num_tokens": 2112,
"size": 5149
} |
{- Byzantine Fault Tolerant Consensus Verification in Agda, version 0.9.
Copyright (c) 2020, 2021, Oracle and/or its affiliates.
Licensed under the Universal Permissive License v 1.0 as shown at https://opensource.oracle.com/licenses/upl
-}
{-# OPTIONS --allow-unsolved-metas #-}
open import Optics.All
open import LibraBFT.Prelude
open import LibraBFT.Base.PKCS
open import LibraBFT.Base.Encode
open import LibraBFT.Base.KVMap as KVMap
open import LibraBFT.Base.Types
open import Data.String using (String)
-- This module defines types for an out-of-date implementation, based
-- on a previous version of LibraBFT. It will be updated to model a
-- more recent version in future.
--
-- One important trick here is that the RoundManager type separayes
-- types that /define/ the EpochConfig and types that /use/ the
-- /EpochConfig/. The advantage of doing this separation can be seen
-- in Util.Util.liftEC, where we define a lifting of a function that
-- does not change the bits that define the EpochConfig into the whole
-- state. This enables a more elegant approach for reasoning about
-- functions that do not change parts of the state responsible for
-- defining the epoch config. However, the separation is not perfect,
-- so sometimes fields may be modified in EpochIndep even though there
-- is no epoch change.
module LibraBFT.Impl.Consensus.Types where
open import LibraBFT.Impl.Base.Types public
open import LibraBFT.Impl.NetworkMsg public
open import LibraBFT.Abstract.Types.EpochConfig UID NodeId public
open import LibraBFT.Impl.Consensus.Types.EpochIndep public
open import LibraBFT.Impl.Consensus.Types.EpochDep public
record EpochState : Set where
constructor EpochState∙new
field
₋esEpoch : Epoch
₋esVerifier : ValidatorVerifier
open EpochState public
unquoteDecl esEpoch esVerifier = mkLens (quote EpochState)
(esEpoch ∷ esVerifier ∷ [])
-- The parts of the state of a peer that are used to
-- define the EpochConfig are the SafetyRules and ValidatorVerifier:
record RoundManagerEC : Set where
constructor RoundManagerEC∙new
field
₋rmEpochState : EpochState
₋rmSafetyRules : SafetyRules
open RoundManagerEC public
unquoteDecl rmEpochState rmSafetyRules = mkLens (quote RoundManagerEC)
(rmEpochState ∷ rmSafetyRules ∷ [])
rmEpoch : Lens RoundManagerEC Epoch
rmEpoch = rmEpochState ∙ esEpoch
rmLastVotedRound : Lens RoundManagerEC Round
rmLastVotedRound = rmSafetyRules ∙ srPersistentStorage ∙ pssSafetyData ∙ sdLastVotedRound
-- We need enough authors to withstand the desired number of
-- byzantine failures. We enforce this with a predicate over
-- 'RoundManagerEC'.
RoundManagerEC-correct : RoundManagerEC → Set
RoundManagerEC-correct rmec =
let numAuthors = kvm-size (rmec ^∙ rmEpochState ∙ esVerifier ∙ vvAddressToValidatorInfo)
qsize = rmec ^∙ rmEpochState ∙ esVerifier ∙ vvQuorumVotingPower
bizF = numAuthors ∸ qsize
in suc (3 * bizF) ≤ numAuthors
RoundManagerEC-correct-≡ : (rmec1 : RoundManagerEC)
→ (rmec2 : RoundManagerEC)
→ (rmec1 ^∙ rmEpochState ∙ esVerifier) ≡ (rmec2 ^∙ rmEpochState ∙ esVerifier)
→ RoundManagerEC-correct rmec1
→ RoundManagerEC-correct rmec2
RoundManagerEC-correct-≡ rmec1 rmec2 refl = id
-- Given a well-formed set of definitions that defines an EpochConfig,
-- α-EC will compute this EpochConfig by abstracting away the unecessary
-- pieces from RoundManagerEC.
-- TODO-2: update and complete when definitions are updated to more recent version
α-EC : Σ RoundManagerEC RoundManagerEC-correct → EpochConfig
α-EC (rmec , ok) =
let numAuthors = kvm-size (rmec ^∙ rmEpochState ∙ esVerifier ∙ vvAddressToValidatorInfo)
qsize = rmec ^∙ rmEpochState ∙ esVerifier ∙ vvQuorumVotingPower
bizF = numAuthors ∸ qsize
in (EpochConfig∙new {! someHash?!}
(rmec ^∙ rmEpoch) numAuthors {!!} {!!} {!!} {!!} {!!} {!!} {!!} {!!})
postulate
α-EC-≡ : (rmec1 : RoundManagerEC)
→ (rmec2 : RoundManagerEC)
→ (vals≡ : rmec1 ^∙ rmEpochState ∙ esVerifier ≡ rmec2 ^∙ rmEpochState ∙ esVerifier)
→ rmec1 ^∙ rmEpoch ≡ rmec2 ^∙ rmEpoch
→ (rmec1-corr : RoundManagerEC-correct rmec1)
→ α-EC (rmec1 , rmec1-corr) ≡ α-EC (rmec2 , RoundManagerEC-correct-≡ rmec1 rmec2 vals≡ rmec1-corr)
{-
α-EC-≡ rmec1 rmec2 refl refl rmec1-corr = refl
-}
-- Just in case RoundManager is at a higher level in future
ℓ-RoundManager : Level
ℓ-RoundManager = 0ℓ
-- Finally, the RoundManager is split in two pieces: those that are used to make an EpochConfig
-- versus those that use an EpochConfig. The reason is that the *abstract* EpochConfig is a
-- function of some parts of the RoundManager (₋rmEC), and some parts depend on the abstract
-- EpochConfig. For example, ₋btIdToQuorumCert carries a proof that the QuorumCert is valid (for
-- the abstract EpochConfig).
record RoundManager : Set ℓ-RoundManager where
constructor RoundManager∙new
field
₋rmEC : RoundManagerEC
₋rmEC-correct : RoundManagerEC-correct ₋rmEC
₋rmWithEC : RoundManagerWithEC (α-EC (₋rmEC , ₋rmEC-correct))
-- If we want to add pieces that neither contribute to the
-- construction of the EC nor need one, they should be defined in
-- RoundManager directly
open RoundManager public
α-EC-RM : RoundManager → EpochConfig
α-EC-RM rm = α-EC ((₋rmEC rm) , (₋rmEC-correct rm))
₋rmHighestQC : (rm : RoundManager) → QuorumCert
₋rmHighestQC rm = ₋btHighestQuorumCert ((₋rmWithEC rm) ^∙ (lBlockTree (α-EC-RM rm)))
rmHighestQC : Lens RoundManager QuorumCert
rmHighestQC = mkLens' ₋rmHighestQC
(λ (RoundManager∙new ec ecc (RoundManagerWithEC∙new (BlockStore∙new bsInner))) qc
→ RoundManager∙new ec ecc (RoundManagerWithEC∙new (BlockStore∙new (record bsInner {₋btHighestQuorumCert = qc}))))
₋rmHighestCommitQC : (rm : RoundManager) → QuorumCert
₋rmHighestCommitQC rm = ₋btHighestCommitCert ((₋rmWithEC rm) ^∙ (lBlockTree (α-EC-RM rm)))
rmHighestCommitQC : Lens RoundManager QuorumCert
rmHighestCommitQC = mkLens' ₋rmHighestCommitQC
(λ (RoundManager∙new ec ecc (RoundManagerWithEC∙new (BlockStore∙new bsInner))) qc
→ RoundManager∙new ec ecc (RoundManagerWithEC∙new (BlockStore∙new (record bsInner {₋btHighestCommitCert = qc}))))
| {
"alphanum_fraction": 0.6927340824,
"avg_line_length": 47.3404255319,
"ext": "agda",
"hexsha": "c11ec29679f7c9cc1ad8dcff1c096ee0ca239f14",
"lang": "Agda",
"max_forks_count": null,
"max_forks_repo_forks_event_max_datetime": null,
"max_forks_repo_forks_event_min_datetime": null,
"max_forks_repo_head_hexsha": "71aa2168e4875ffdeece9ba7472ee3cee5fa9084",
"max_forks_repo_licenses": [
"UPL-1.0"
],
"max_forks_repo_name": "cwjnkins/bft-consensus-agda",
"max_forks_repo_path": "LibraBFT/Impl/Consensus/Types.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "71aa2168e4875ffdeece9ba7472ee3cee5fa9084",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"UPL-1.0"
],
"max_issues_repo_name": "cwjnkins/bft-consensus-agda",
"max_issues_repo_path": "LibraBFT/Impl/Consensus/Types.agda",
"max_line_length": 139,
"max_stars_count": null,
"max_stars_repo_head_hexsha": "71aa2168e4875ffdeece9ba7472ee3cee5fa9084",
"max_stars_repo_licenses": [
"UPL-1.0"
],
"max_stars_repo_name": "cwjnkins/bft-consensus-agda",
"max_stars_repo_path": "LibraBFT/Impl/Consensus/Types.agda",
"max_stars_repo_stars_event_max_datetime": null,
"max_stars_repo_stars_event_min_datetime": null,
"num_tokens": 1929,
"size": 6675
} |
{-# OPTIONS --cubical-compatible #-}
module Common.Integer where
open import Agda.Builtin.Int public renaming (Int to Integer)
| {
"alphanum_fraction": 0.765625,
"avg_line_length": 25.6,
"ext": "agda",
"hexsha": "53a1261c5eda07ba0d6fc89957432172bd1bc1b9",
"lang": "Agda",
"max_forks_count": null,
"max_forks_repo_forks_event_max_datetime": null,
"max_forks_repo_forks_event_min_datetime": null,
"max_forks_repo_head_hexsha": "98c9382a59f707c2c97d75919e389fc2a783ac75",
"max_forks_repo_licenses": [
"BSD-2-Clause"
],
"max_forks_repo_name": "KDr2/agda",
"max_forks_repo_path": "test/Common/Integer.agda",
"max_issues_count": 6,
"max_issues_repo_head_hexsha": "98c9382a59f707c2c97d75919e389fc2a783ac75",
"max_issues_repo_issues_event_max_datetime": "2021-11-24T08:31:10.000Z",
"max_issues_repo_issues_event_min_datetime": "2021-10-18T08:12:24.000Z",
"max_issues_repo_licenses": [
"BSD-2-Clause"
],
"max_issues_repo_name": "KDr2/agda",
"max_issues_repo_path": "test/Common/Integer.agda",
"max_line_length": 61,
"max_stars_count": null,
"max_stars_repo_head_hexsha": "98c9382a59f707c2c97d75919e389fc2a783ac75",
"max_stars_repo_licenses": [
"BSD-2-Clause"
],
"max_stars_repo_name": "KDr2/agda",
"max_stars_repo_path": "test/Common/Integer.agda",
"max_stars_repo_stars_event_max_datetime": null,
"max_stars_repo_stars_event_min_datetime": null,
"num_tokens": 27,
"size": 128
} |
-- Andreas, 2012-03-30
module Issue593 where
import Common.Level
open import Common.Equality
open import Common.Irrelevance
record Unit : Set where
constructor unit
bla6 : (F : Unit -> Set) ->
let X : Unit -> Unit -> Set
X = _
in (z : Unit) -> X z z ≡ F z
bla6 F z = refl
-- non-linearity for singleton types should not matter
bla7 : (F : Unit -> Set) ->
let X : Set
X = _
in (z : Unit) -> X ≡ F z
bla7 F z = refl
-- should eta expand z to unit
-- * a more involved singleton type:
record R (A : Set) : Set where
constructor r
field
f1 : A -> Unit
f2 : A
Sing : Set1
Sing = (A : Set) -> A -> R (A -> Unit)
test : (F : Sing -> Set) ->
let X : Set
X = _
in (z : Sing) -> X ≡ F z
test F z = refl
-- * something with irrelevance
Sing' : Set1
Sing' = (A : Set) -> A -> R (Squash A)
test' : (F : Sing' -> Set) ->
let X : Sing' -> Sing' -> Set
X = _
in (z : Sing') -> X z z ≡ F z
test' F z = refl
-- non-linearity should not matter
| {
"alphanum_fraction": 0.5616161616,
"avg_line_length": 18.679245283,
"ext": "agda",
"hexsha": "acda8483cdc9af917b55d4c4e4ddb6863854b9cf",
"lang": "Agda",
"max_forks_count": 371,
"max_forks_repo_forks_event_max_datetime": "2022-03-30T19:00:30.000Z",
"max_forks_repo_forks_event_min_datetime": "2015-01-03T14:04:08.000Z",
"max_forks_repo_head_hexsha": "231d6ad8e77b67ff8c4b1cb35a6c31ccd988c3e9",
"max_forks_repo_licenses": [
"BSD-3-Clause"
],
"max_forks_repo_name": "Agda-zh/agda",
"max_forks_repo_path": "test/Succeed/Issue593.agda",
"max_issues_count": 4066,
"max_issues_repo_head_hexsha": "ed8ac6f4062ea8a20fa0f62d5db82d4e68278338",
"max_issues_repo_issues_event_max_datetime": "2022-03-31T21:14:49.000Z",
"max_issues_repo_issues_event_min_datetime": "2015-01-10T11:24:51.000Z",
"max_issues_repo_licenses": [
"BSD-3-Clause"
],
"max_issues_repo_name": "shlevy/agda",
"max_issues_repo_path": "test/Succeed/Issue593.agda",
"max_line_length": 54,
"max_stars_count": 1989,
"max_stars_repo_head_hexsha": "ed8ac6f4062ea8a20fa0f62d5db82d4e68278338",
"max_stars_repo_licenses": [
"BSD-3-Clause"
],
"max_stars_repo_name": "shlevy/agda",
"max_stars_repo_path": "test/Succeed/Issue593.agda",
"max_stars_repo_stars_event_max_datetime": "2022-03-30T18:20:48.000Z",
"max_stars_repo_stars_event_min_datetime": "2015-01-09T23:51:16.000Z",
"num_tokens": 344,
"size": 990
} |
-- Basic intuitionistic modal logic S4, without ∨, ⊥, or ◇.
-- Hilbert-style formalisation of closed syntax.
-- Sequences of terms.
module BasicIS4.Syntax.ClosedHilbertSequential where
open import BasicIS4.Syntax.Common public
-- Derivations.
infix 3 ⊦⊢_
data ⊦⊢_ : Cx Ty → Set where
nil : ⊦⊢ ∅
mp : ∀ {Ξ A B} → A ▻ B ∈ Ξ → A ∈ Ξ → ⊦⊢ Ξ → ⊦⊢ Ξ , B
ci : ∀ {Ξ A} → ⊦⊢ Ξ → ⊦⊢ Ξ , A ▻ A
ck : ∀ {Ξ A B} → ⊦⊢ Ξ → ⊦⊢ Ξ , A ▻ B ▻ A
cs : ∀ {Ξ A B C} → ⊦⊢ Ξ → ⊦⊢ Ξ , (A ▻ B ▻ C) ▻ (A ▻ B) ▻ A ▻ C
nec : ∀ {Ξ Ξ′ A} → ⊦⊢ Ξ′ , A → ⊦⊢ Ξ → ⊦⊢ Ξ , □ A
cdist : ∀ {Ξ A B} → ⊦⊢ Ξ → ⊦⊢ Ξ , □ (A ▻ B) ▻ □ A ▻ □ B
cup : ∀ {Ξ A} → ⊦⊢ Ξ → ⊦⊢ Ξ , □ A ▻ □ □ A
cdown : ∀ {Ξ A} → ⊦⊢ Ξ → ⊦⊢ Ξ , □ A ▻ A
cpair : ∀ {Ξ A B} → ⊦⊢ Ξ → ⊦⊢ Ξ , A ▻ B ▻ A ∧ B
cfst : ∀ {Ξ A B} → ⊦⊢ Ξ → ⊦⊢ Ξ , A ∧ B ▻ A
csnd : ∀ {Ξ A B} → ⊦⊢ Ξ → ⊦⊢ Ξ , A ∧ B ▻ B
unit : ∀ {Ξ} → ⊦⊢ Ξ → ⊦⊢ Ξ , ⊤
infix 3 ⊢_
⊢_ : Ty → Set
⊢ A = ∃ (λ Ξ → ⊦⊢ Ξ , A)
-- Concatenation of derivations.
_⧺⊦_ : ∀ {Ξ Ξ′} → ⊦⊢ Ξ → ⊦⊢ Ξ′ → ⊦⊢ Ξ ⧺ Ξ′
us ⧺⊦ nil = us
us ⧺⊦ mp i j ts = mp (mono∈ weak⊆⧺₂ i) (mono∈ weak⊆⧺₂ j) (us ⧺⊦ ts)
us ⧺⊦ ci ts = ci (us ⧺⊦ ts)
us ⧺⊦ ck ts = ck (us ⧺⊦ ts)
us ⧺⊦ cs ts = cs (us ⧺⊦ ts)
us ⧺⊦ nec ss ts = nec ss (us ⧺⊦ ts)
us ⧺⊦ cdist ts = cdist (us ⧺⊦ ts)
us ⧺⊦ cup ts = cup (us ⧺⊦ ts)
us ⧺⊦ cdown ts = cdown (us ⧺⊦ ts)
us ⧺⊦ cpair ts = cpair (us ⧺⊦ ts)
us ⧺⊦ cfst ts = cfst (us ⧺⊦ ts)
us ⧺⊦ csnd ts = csnd (us ⧺⊦ ts)
us ⧺⊦ unit ts = unit (us ⧺⊦ ts)
-- Modus ponens and necessitation in expanded form.
app : ∀ {A B} → ⊢ A ▻ B → ⊢ A → ⊢ B
app {A} {B} (Ξ , ts) (Ξ′ , us) = Ξ″ , vs
where Ξ″ = (Ξ′ , A) ⧺ (Ξ , A ▻ B)
vs = mp top (mono∈ (weak⊆⧺₁ (Ξ , A ▻ B)) top) (us ⧺⊦ ts)
box : ∀ {A} → ⊢ A → ⊢ □ A
box (Ξ , ts) = ∅ , nec ts nil
| {
"alphanum_fraction": 0.4087631725,
"avg_line_length": 30.05,
"ext": "agda",
"hexsha": "71c16210f42099581613e97b6a59afa058bcd57b",
"lang": "Agda",
"max_forks_count": null,
"max_forks_repo_forks_event_max_datetime": null,
"max_forks_repo_forks_event_min_datetime": null,
"max_forks_repo_head_hexsha": "fcd187db70f0a39b894fe44fad0107f61849405c",
"max_forks_repo_licenses": [
"X11"
],
"max_forks_repo_name": "mietek/hilbert-gentzen",
"max_forks_repo_path": "BasicIS4/Syntax/ClosedHilbertSequential.agda",
"max_issues_count": 1,
"max_issues_repo_head_hexsha": "fcd187db70f0a39b894fe44fad0107f61849405c",
"max_issues_repo_issues_event_max_datetime": "2018-06-10T09:11:22.000Z",
"max_issues_repo_issues_event_min_datetime": "2018-06-10T09:11:22.000Z",
"max_issues_repo_licenses": [
"X11"
],
"max_issues_repo_name": "mietek/hilbert-gentzen",
"max_issues_repo_path": "BasicIS4/Syntax/ClosedHilbertSequential.agda",
"max_line_length": 67,
"max_stars_count": 29,
"max_stars_repo_head_hexsha": "fcd187db70f0a39b894fe44fad0107f61849405c",
"max_stars_repo_licenses": [
"X11"
],
"max_stars_repo_name": "mietek/hilbert-gentzen",
"max_stars_repo_path": "BasicIS4/Syntax/ClosedHilbertSequential.agda",
"max_stars_repo_stars_event_max_datetime": "2022-01-01T10:29:18.000Z",
"max_stars_repo_stars_event_min_datetime": "2016-07-03T18:51:56.000Z",
"num_tokens": 1146,
"size": 1803
} |
{-# OPTIONS --safe #-} --without-K #-}
import Data.Product as Product
import Data.Product.Properties as Productₚ
import Data.Nat as Nat
import Data.Vec as Vec
import Data.Vec.Properties as Vecₚ
import Data.Fin as Fin
import Data.Vec.Relation.Unary.All as All
open Nat using (ℕ; zero; suc)
open Vec using (Vec; []; _∷_)
open All using (All; []; _∷_)
open Fin using (Fin ; zero ; suc)
open Product using (_,_)
import PiCalculus.Syntax
open PiCalculus.Syntax.Scoped
open import PiCalculus.Semantics
open import PiCalculus.LinearTypeSystem.Algebras
module PiCalculus.LinearTypeSystem.Weakening (Ω : Algebras) where
open Algebras Ω
open import PiCalculus.LinearTypeSystem.ContextLemmas Ω
open import PiCalculus.LinearTypeSystem Ω
private
variable
n : ℕ
i j : Fin n
idx idx' : Idx
idxs : Idxs n
P Q : Scoped n
∋-weaken : {γ : PreCtx n} {Γ Θ : Ctx idxs} {t t' : Type} {xs : Usage idx ²} {xs' : Usage idx' ²}
→ (j : Fin (suc n))
→ γ ; Γ ∋[ i ] t' ; xs' ▹ Θ
→ Vec.insert γ j t ; ctx-insert j xs Γ ∋[ Fin.punchIn j i ] t' ; xs' ▹ ctx-insert j xs Θ
∋-weaken zero x = there x
∋-weaken (suc i) (zero , zero xyz) = zero , zero xyz
∋-weaken (suc i) (suc t , suc x) = there (∋-weaken i (t , x))
⊢-weaken : {P : Scoped n} {γ : PreCtx n} {Γ Θ : Ctx idxs} {t : Type} {xs : Usage idx ²}
→ (j : Fin (suc n))
→ γ ; Γ ⊢ P ▹ Θ
→ Vec.insert γ j t ; ctx-insert j xs Γ ⊢ lift j P ▹ ctx-insert j xs Θ
⊢-weaken j 𝟘 = 𝟘
⊢-weaken j (ν t m μ ⊢P) = ν t m μ (⊢-weaken (suc j) ⊢P)
⊢-weaken j (⊢P ∥ ⊢Q) = ⊢-weaken j ⊢P ∥ ⊢-weaken j ⊢Q
⊢-weaken j (x ⦅⦆ ⊢P) = ∋-weaken j x ⦅⦆ ⊢-weaken (suc j) ⊢P
⊢-weaken j (x ⟨ y ⟩ ⊢P) = ∋-weaken j x ⟨ ∋-weaken j y ⟩ ⊢-weaken j ⊢P
| {
"alphanum_fraction": 0.5951025057,
"avg_line_length": 33.7692307692,
"ext": "agda",
"hexsha": "f344101b866019c7fe0ef657b415bcc1a1ed6973",
"lang": "Agda",
"max_forks_count": 3,
"max_forks_repo_forks_event_max_datetime": "2022-03-14T16:24:07.000Z",
"max_forks_repo_forks_event_min_datetime": "2021-01-25T13:57:13.000Z",
"max_forks_repo_head_hexsha": "0fc3cf6bcc0cd07d4511dbe98149ac44e6a38b1a",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "guilhermehas/typing-linear-pi",
"max_forks_repo_path": "src/PiCalculus/LinearTypeSystem/Weakening.agda",
"max_issues_count": 1,
"max_issues_repo_head_hexsha": "0fc3cf6bcc0cd07d4511dbe98149ac44e6a38b1a",
"max_issues_repo_issues_event_max_datetime": "2022-03-15T09:16:14.000Z",
"max_issues_repo_issues_event_min_datetime": "2022-03-15T09:16:14.000Z",
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "guilhermehas/typing-linear-pi",
"max_issues_repo_path": "src/PiCalculus/LinearTypeSystem/Weakening.agda",
"max_line_length": 97,
"max_stars_count": 26,
"max_stars_repo_head_hexsha": "0fc3cf6bcc0cd07d4511dbe98149ac44e6a38b1a",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "guilhermehas/typing-linear-pi",
"max_stars_repo_path": "src/PiCalculus/LinearTypeSystem/Weakening.agda",
"max_stars_repo_stars_event_max_datetime": "2022-03-14T15:18:23.000Z",
"max_stars_repo_stars_event_min_datetime": "2020-05-02T23:32:11.000Z",
"num_tokens": 715,
"size": 1756
} |
{-# OPTIONS --without-K --safe #-}
module Categories.Functor.Equivalence where
-- A 'strict' equality relation for Functors.
open import Level
open import Data.Product using (Σ; curry) renaming (_,_ to _,,_)
open import Relation.Binary.PropositionalEquality as ≡
open import Relation.Binary using (IsEquivalence)
open import Function using (_$_) renaming (_∘_ to _⊚_)
open import Categories.Category using (Category; _[_,_]; _[_≈_])
open import Categories.Category.Product
open import Categories.Functor using (Functor; _∘F_) renaming (id to idF)
open import Categories.Functor.Bifunctor
open import Categories.Functor.Properties using ([_]-resp-square)
open import Categories.NaturalTransformation using (ntHelper)
import Categories.Morphism as Morphism
import Categories.Morphism.HeterogeneousIdentity as HId
import Categories.Morphism.HeterogeneousIdentity.Properties as HIdProps
import Categories.Morphism.IsoEquiv as IsoEquiv
import Categories.Morphism.Reasoning as MorphismReasoning
import Categories.NaturalTransformation.NaturalIsomorphism as NatIso
private
variable
o ℓ e o′ ℓ′ e′ o″ ℓ″ e″ o‴ ℓ‴ e‴ : Level
-- "Strict" equality of Functors.
--
-- It's helpful to think of a functor equality (P : F ≡F G) as a
-- special natural isomorphism where every component (hid $ eq₀ P X)
-- is a 'heterogeneous' identity.
infix 4 _≡F_
record _≡F_ {C : Category o ℓ e}
{D : Category o′ ℓ′ e′}
(F G : Functor C D) : Set (ℓ ⊔ o ⊔ o′ ⊔ e′) where
private
module C = Category C
module D = Category D
module F = Functor F
module G = Functor G
open F using (F₀; F₁)
open G using () renaming (F₀ to G₀; F₁ to G₁)
open HId D
field
eq₀ : ∀ X → F₀ X ≡ G₀ X
eq₁ : ∀ {X Y} (f : C [ X , Y ]) →
D.CommutativeSquare (F₁ f) (hid $ eq₀ X) (hid $ eq₀ Y) (G₁ f)
eq₀⁻¹ : ∀ X → G₀ X ≡ F₀ X
eq₀⁻¹ X = sym $ eq₀ X
eq₁⁻¹ : ∀ {X Y} (f : C [ X , Y ]) →
D.CommutativeSquare (G₁ f) (hid $ eq₀⁻¹ X) (hid $ eq₀⁻¹ Y) (F₁ f)
eq₁⁻¹ {X} {Y} f = begin
τ⁻¹ Y ∘ G₁ f ≈˘⟨ identityʳ ⟩
(τ⁻¹ Y ∘ G₁ f) ∘ id ≈˘⟨ ∘-resp-≈ʳ $ hid-symʳ _ ⟩
(τ⁻¹ Y ∘ G₁ f) ∘ (τ X ∘ τ⁻¹ X) ≈⟨ assoc ⟩
τ⁻¹ Y ∘ (G₁ f ∘ (τ X ∘ τ⁻¹ X)) ≈˘⟨ ∘-resp-≈ʳ assoc ⟩
τ⁻¹ Y ∘ ((G₁ f ∘ τ X) ∘ τ⁻¹ X) ≈˘⟨ ∘-resp-≈ʳ $ ∘-resp-≈ˡ $ eq₁ f ⟩
τ⁻¹ Y ∘ ((τ Y ∘ F₁ f) ∘ τ⁻¹ X) ≈˘⟨ assoc ⟩
(τ⁻¹ Y ∘ (τ Y ∘ F₁ f)) ∘ τ⁻¹ X ≈˘⟨ ∘-resp-≈ˡ assoc ⟩
((τ⁻¹ Y ∘ τ Y) ∘ F₁ f) ∘ τ⁻¹ X ≈⟨ ∘-resp-≈ˡ $ ∘-resp-≈ˡ $ hid-symˡ _ ⟩
(id ∘ F₁ f) ∘ τ⁻¹ X ≈⟨ ∘-resp-≈ˡ identityˡ ⟩
F₁ f ∘ τ⁻¹ X ∎
where
τ = λ X → hid $ eq₀ X
τ⁻¹ = λ X → hid $ eq₀⁻¹ X
open D
open HomReasoning
open NatIso using (_≃_)
-- the family (hid eq₀) is a natural isomorphism
natIso : F ≃ G
natIso = record
{ F⇒G = ntHelper record { η = hid ⊚ eq₀ ; commute = eq₁ }
; F⇐G = ntHelper record { η = hid ⊚ eq₀⁻¹ ; commute = eq₁⁻¹ }
; iso = λ X → hid-iso $ eq₀ X
}
module _ {C : Category o ℓ e} {D : Category o′ ℓ′ e′} where
open Functor
open Category D
open HomReasoning hiding (refl; trans)
open MorphismReasoning D
open HId D
open _≡F_
-- Strict functor equality is an equivalence.
≡F-equiv : IsEquivalence (_≡F_ {C = C} {D})
≡F-equiv = record
{ refl = record { eq₀ = λ _ → refl ; eq₁ = λ _ → id-comm-sym }
; sym = λ F≡G → record { eq₀ = eq₀⁻¹ F≡G ; eq₁ = eq₁⁻¹ F≡G }
; trans = λ {F G H} F≡G G≡H → record
{ eq₀ = λ X → trans (eq₀ F≡G X) (eq₀ G≡H X)
; eq₁ = λ {X} {Y} f → begin
hid (trans (eq₀ F≡G Y) (eq₀ G≡H Y)) ∘ F₁ F f
≈˘⟨ ∘-resp-≈ˡ (hid-trans _ _) ⟩
(hid (eq₀ G≡H Y) ∘ hid (eq₀ F≡G Y)) ∘ F₁ F f
≈⟨ glue (eq₁ G≡H f) (eq₁ F≡G f) ⟩
F₁ H f ∘ (hid (eq₀ G≡H X) ∘ hid (eq₀ F≡G X))
≈⟨ ∘-resp-≈ʳ (hid-trans _ _) ⟩
F₁ H f ∘ hid (trans (eq₀ F≡G X) (eq₀ G≡H X))
∎
}
}
≡F-identityˡ : {F : Functor C D} → idF ∘F F ≡F F
≡F-identityˡ = record { eq₀ = λ _ → refl ; eq₁ = λ _ → id-comm-sym }
≡F-identityʳ : {F : Functor C D} → F ∘F idF ≡F F
≡F-identityʳ = record { eq₀ = λ _ → refl ; eq₁ = λ _ → id-comm-sym }
module _ {C : Category o ℓ e} where
open MorphismReasoning C
≡F-identity² : idF ∘F idF ≡F idF {C = C}
≡F-identity² = record { eq₀ = λ _ → refl ; eq₁ = λ _ → id-comm-sym }
module _ {C : Category o ℓ e} {D : Category o′ ℓ′ e′}
{E : Category o″ ℓ″ e″}
where
open Functor
open Category E
open HomReasoning hiding (refl; trans)
open MorphismReasoning E
open HId
open HIdProps
open _≡F_
∘F-resp-≡F : {H I : Functor D E} {F G : Functor C D} →
H ≡F I → F ≡F G → H ∘F F ≡F I ∘F G
∘F-resp-≡F {H} {I} {F} {G} H≡I F≡G = record
{ eq₀ = λ X → trans (HF≡HG X) (HG≡IG X)
; eq₁ = λ {X Y} f → begin
hid E (trans (HF≡HG Y) (HG≡IG Y)) ∘ F₁ H (F₁ F f)
≈˘⟨ ∘-resp-≈ˡ (hid-trans E _ _) ⟩
(hid E (HG≡IG Y) ∘ hid E (HF≡HG Y)) ∘ F₁ H (F₁ F f)
≈˘⟨ ∘-resp-≈ˡ $ ∘-resp-≈ʳ (F-hid H (eq₀ F≡G Y)) ⟩
(hid E (HG≡IG Y) ∘ F₁ H (hid D (eq₀ F≡G Y))) ∘ F₁ H (F₁ F f)
≈⟨ glue (eq₁ H≡I (F₁ G f)) ([ H ]-resp-square (eq₁ F≡G f)) ⟩
F₁ I (F₁ G f) ∘ (hid E (HG≡IG X) ∘ F₁ H (hid D (eq₀ F≡G X)))
≈⟨ ∘-resp-≈ʳ $ ∘-resp-≈ʳ (F-hid H (eq₀ F≡G X)) ⟩
F₁ I (F₁ G f) ∘ (hid E (HG≡IG X) ∘ hid E (HF≡HG X))
≈⟨ ∘-resp-≈ʳ (hid-trans E _ _) ⟩
F₁ I (F₁ G f) ∘ hid E (trans (HF≡HG X) (HG≡IG X))
∎
}
where
HF≡HG = λ X → cong (F₀ H) (eq₀ F≡G X)
HG≡IG = λ X → eq₀ H≡I (F₀ G X)
module _ {B : Category o ℓ e} {C : Category o′ ℓ′ e′}
{D : Category o″ ℓ″ e″} {E : Category o‴ ℓ‴ e‴}
where
open Functor
open Category E
open MorphismReasoning E
open _≡F_
≡F-assoc : {F : Functor B C} {G : Functor C D} {H : Functor D E} →
(H ∘F G) ∘F F ≡F H ∘F (G ∘F F)
≡F-assoc = record { eq₀ = λ _ → refl ; eq₁ = λ _ → id-comm-sym }
≡F-sym-assoc : {F : Functor B C} {G : Functor C D} {H : Functor D E} →
H ∘F (G ∘F F) ≡F (H ∘F G) ∘F F
≡F-sym-assoc = record { eq₀ = λ _ → refl ; eq₁ = λ _ → id-comm-sym }
| {
"alphanum_fraction": 0.532547246,
"avg_line_length": 34.5865921788,
"ext": "agda",
"hexsha": "b1eb71c5b88e14b3ac067cbd587cdd73e193e28c",
"lang": "Agda",
"max_forks_count": null,
"max_forks_repo_forks_event_max_datetime": null,
"max_forks_repo_forks_event_min_datetime": null,
"max_forks_repo_head_hexsha": "6ebc1349ee79669c5c496dcadd551d5bbefd1972",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "Taneb/agda-categories",
"max_forks_repo_path": "Categories/Functor/Equivalence.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "6ebc1349ee79669c5c496dcadd551d5bbefd1972",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "Taneb/agda-categories",
"max_issues_repo_path": "Categories/Functor/Equivalence.agda",
"max_line_length": 81,
"max_stars_count": null,
"max_stars_repo_head_hexsha": "6ebc1349ee79669c5c496dcadd551d5bbefd1972",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "Taneb/agda-categories",
"max_stars_repo_path": "Categories/Functor/Equivalence.agda",
"max_stars_repo_stars_event_max_datetime": null,
"max_stars_repo_stars_event_min_datetime": null,
"num_tokens": 2754,
"size": 6191
} |
------------------------------------------------------------------------------
-- Common properties for the alternating bit protocol
------------------------------------------------------------------------------
{-# OPTIONS --exact-split #-}
{-# OPTIONS --no-sized-types #-}
{-# OPTIONS --no-universe-polymorphism #-}
{-# OPTIONS --without-K #-}
module FOTC.Program.ABP.PropertiesI where
open import FOTC.Base
open import FOTC.Program.ABP.ABP
------------------------------------------------------------------------------
-- Congruence properties
awaitCong₄ : ∀ {b i is ds₁ ds₂} → ds₁ ≡ ds₂ →
await b i is ds₁ ≡ await b i is ds₂
awaitCong₄ refl = refl
corruptCong : ∀ {os₁ os₂} → os₁ ≡ os₂ → corrupt os₁ ≡ corrupt os₂
corruptCong refl = refl
| {
"alphanum_fraction": 0.4443053817,
"avg_line_length": 33.2916666667,
"ext": "agda",
"hexsha": "106b204f6c9ad658a6b7b7b16272a8553bf07330",
"lang": "Agda",
"max_forks_count": 3,
"max_forks_repo_forks_event_max_datetime": "2018-03-14T08:50:00.000Z",
"max_forks_repo_forks_event_min_datetime": "2016-09-19T14:18:30.000Z",
"max_forks_repo_head_hexsha": "2fc9f2b81052a2e0822669f02036c5750371b72d",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "asr/fotc",
"max_forks_repo_path": "src/fot/FOTC/Program/ABP/PropertiesI.agda",
"max_issues_count": 2,
"max_issues_repo_head_hexsha": "2fc9f2b81052a2e0822669f02036c5750371b72d",
"max_issues_repo_issues_event_max_datetime": "2017-01-01T14:34:26.000Z",
"max_issues_repo_issues_event_min_datetime": "2016-10-12T17:28:16.000Z",
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "asr/fotc",
"max_issues_repo_path": "src/fot/FOTC/Program/ABP/PropertiesI.agda",
"max_line_length": 78,
"max_stars_count": 11,
"max_stars_repo_head_hexsha": "2fc9f2b81052a2e0822669f02036c5750371b72d",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "asr/fotc",
"max_stars_repo_path": "src/fot/FOTC/Program/ABP/PropertiesI.agda",
"max_stars_repo_stars_event_max_datetime": "2021-09-12T16:09:54.000Z",
"max_stars_repo_stars_event_min_datetime": "2015-09-03T20:53:42.000Z",
"num_tokens": 165,
"size": 799
} |
module Text.Greek.SBLGNT.John where
open import Data.List
open import Text.Greek.Bible
open import Text.Greek.Script
open import Text.Greek.Script.Unicode
ΚΑΤΑ-ΙΩΑΝΝΗΝ : List (Word)
ΚΑΤΑ-ΙΩΑΝΝΗΝ =
word (Ἐ ∷ ν ∷ []) "John.1.1"
∷ word (ἀ ∷ ρ ∷ χ ∷ ῇ ∷ []) "John.1.1"
∷ word (ἦ ∷ ν ∷ []) "John.1.1"
∷ word (ὁ ∷ []) "John.1.1"
∷ word (∙λ ∷ ό ∷ γ ∷ ο ∷ ς ∷ []) "John.1.1"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.1"
∷ word (ὁ ∷ []) "John.1.1"
∷ word (∙λ ∷ ό ∷ γ ∷ ο ∷ ς ∷ []) "John.1.1"
∷ word (ἦ ∷ ν ∷ []) "John.1.1"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.1.1"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.1.1"
∷ word (θ ∷ ε ∷ ό ∷ ν ∷ []) "John.1.1"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.1"
∷ word (θ ∷ ε ∷ ὸ ∷ ς ∷ []) "John.1.1"
∷ word (ἦ ∷ ν ∷ []) "John.1.1"
∷ word (ὁ ∷ []) "John.1.1"
∷ word (∙λ ∷ ό ∷ γ ∷ ο ∷ ς ∷ []) "John.1.1"
∷ word (ο ∷ ὗ ∷ τ ∷ ο ∷ ς ∷ []) "John.1.2"
∷ word (ἦ ∷ ν ∷ []) "John.1.2"
∷ word (ἐ ∷ ν ∷ []) "John.1.2"
∷ word (ἀ ∷ ρ ∷ χ ∷ ῇ ∷ []) "John.1.2"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.1.2"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.1.2"
∷ word (θ ∷ ε ∷ ό ∷ ν ∷ []) "John.1.2"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ α ∷ []) "John.1.3"
∷ word (δ ∷ ι ∷ []) "John.1.3"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.1.3"
∷ word (ἐ ∷ γ ∷ έ ∷ ν ∷ ε ∷ τ ∷ ο ∷ []) "John.1.3"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.3"
∷ word (χ ∷ ω ∷ ρ ∷ ὶ ∷ ς ∷ []) "John.1.3"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.1.3"
∷ word (ἐ ∷ γ ∷ έ ∷ ν ∷ ε ∷ τ ∷ ο ∷ []) "John.1.3"
∷ word (ο ∷ ὐ ∷ δ ∷ ὲ ∷ []) "John.1.3"
∷ word (ἕ ∷ ν ∷ []) "John.1.3"
∷ word (ὃ ∷ []) "John.1.3"
∷ word (γ ∷ έ ∷ γ ∷ ο ∷ ν ∷ ε ∷ ν ∷ []) "John.1.3"
∷ word (ἐ ∷ ν ∷ []) "John.1.4"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.1.4"
∷ word (ζ ∷ ω ∷ ὴ ∷ []) "John.1.4"
∷ word (ἦ ∷ ν ∷ []) "John.1.4"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.4"
∷ word (ἡ ∷ []) "John.1.4"
∷ word (ζ ∷ ω ∷ ὴ ∷ []) "John.1.4"
∷ word (ἦ ∷ ν ∷ []) "John.1.4"
∷ word (τ ∷ ὸ ∷ []) "John.1.4"
∷ word (φ ∷ ῶ ∷ ς ∷ []) "John.1.4"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.1.4"
∷ word (ἀ ∷ ν ∷ θ ∷ ρ ∷ ώ ∷ π ∷ ω ∷ ν ∷ []) "John.1.4"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.5"
∷ word (τ ∷ ὸ ∷ []) "John.1.5"
∷ word (φ ∷ ῶ ∷ ς ∷ []) "John.1.5"
∷ word (ἐ ∷ ν ∷ []) "John.1.5"
∷ word (τ ∷ ῇ ∷ []) "John.1.5"
∷ word (σ ∷ κ ∷ ο ∷ τ ∷ ί ∷ ᾳ ∷ []) "John.1.5"
∷ word (φ ∷ α ∷ ί ∷ ν ∷ ε ∷ ι ∷ []) "John.1.5"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.5"
∷ word (ἡ ∷ []) "John.1.5"
∷ word (σ ∷ κ ∷ ο ∷ τ ∷ ί ∷ α ∷ []) "John.1.5"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ []) "John.1.5"
∷ word (ο ∷ ὐ ∷ []) "John.1.5"
∷ word (κ ∷ α ∷ τ ∷ έ ∷ ∙λ ∷ α ∷ β ∷ ε ∷ ν ∷ []) "John.1.5"
∷ word (Ἐ ∷ γ ∷ έ ∷ ν ∷ ε ∷ τ ∷ ο ∷ []) "John.1.6"
∷ word (ἄ ∷ ν ∷ θ ∷ ρ ∷ ω ∷ π ∷ ο ∷ ς ∷ []) "John.1.6"
∷ word (ἀ ∷ π ∷ ε ∷ σ ∷ τ ∷ α ∷ ∙λ ∷ μ ∷ έ ∷ ν ∷ ο ∷ ς ∷ []) "John.1.6"
∷ word (π ∷ α ∷ ρ ∷ ὰ ∷ []) "John.1.6"
∷ word (θ ∷ ε ∷ ο ∷ ῦ ∷ []) "John.1.6"
∷ word (ὄ ∷ ν ∷ ο ∷ μ ∷ α ∷ []) "John.1.6"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.1.6"
∷ word (Ἰ ∷ ω ∷ ά ∷ ν ∷ ν ∷ η ∷ ς ∷ []) "John.1.6"
∷ word (ο ∷ ὗ ∷ τ ∷ ο ∷ ς ∷ []) "John.1.7"
∷ word (ἦ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.1.7"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.1.7"
∷ word (μ ∷ α ∷ ρ ∷ τ ∷ υ ∷ ρ ∷ ί ∷ α ∷ ν ∷ []) "John.1.7"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.1.7"
∷ word (μ ∷ α ∷ ρ ∷ τ ∷ υ ∷ ρ ∷ ή ∷ σ ∷ ῃ ∷ []) "John.1.7"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.1.7"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.1.7"
∷ word (φ ∷ ω ∷ τ ∷ ό ∷ ς ∷ []) "John.1.7"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.1.7"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.1.7"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ σ ∷ ω ∷ σ ∷ ι ∷ ν ∷ []) "John.1.7"
∷ word (δ ∷ ι ∷ []) "John.1.7"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.1.7"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.1.8"
∷ word (ἦ ∷ ν ∷ []) "John.1.8"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ο ∷ ς ∷ []) "John.1.8"
∷ word (τ ∷ ὸ ∷ []) "John.1.8"
∷ word (φ ∷ ῶ ∷ ς ∷ []) "John.1.8"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ []) "John.1.8"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.1.8"
∷ word (μ ∷ α ∷ ρ ∷ τ ∷ υ ∷ ρ ∷ ή ∷ σ ∷ ῃ ∷ []) "John.1.8"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.1.8"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.1.8"
∷ word (φ ∷ ω ∷ τ ∷ ό ∷ ς ∷ []) "John.1.8"
∷ word (ἦ ∷ ν ∷ []) "John.1.9"
∷ word (τ ∷ ὸ ∷ []) "John.1.9"
∷ word (φ ∷ ῶ ∷ ς ∷ []) "John.1.9"
∷ word (τ ∷ ὸ ∷ []) "John.1.9"
∷ word (ἀ ∷ ∙λ ∷ η ∷ θ ∷ ι ∷ ν ∷ ὸ ∷ ν ∷ []) "John.1.9"
∷ word (ὃ ∷ []) "John.1.9"
∷ word (φ ∷ ω ∷ τ ∷ ί ∷ ζ ∷ ε ∷ ι ∷ []) "John.1.9"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ α ∷ []) "John.1.9"
∷ word (ἄ ∷ ν ∷ θ ∷ ρ ∷ ω ∷ π ∷ ο ∷ ν ∷ []) "John.1.9"
∷ word (ἐ ∷ ρ ∷ χ ∷ ό ∷ μ ∷ ε ∷ ν ∷ ο ∷ ν ∷ []) "John.1.9"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.1.9"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.1.9"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ ν ∷ []) "John.1.9"
∷ word (Ἐ ∷ ν ∷ []) "John.1.10"
∷ word (τ ∷ ῷ ∷ []) "John.1.10"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ῳ ∷ []) "John.1.10"
∷ word (ἦ ∷ ν ∷ []) "John.1.10"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.10"
∷ word (ὁ ∷ []) "John.1.10"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ ς ∷ []) "John.1.10"
∷ word (δ ∷ ι ∷ []) "John.1.10"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.1.10"
∷ word (ἐ ∷ γ ∷ έ ∷ ν ∷ ε ∷ τ ∷ ο ∷ []) "John.1.10"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.10"
∷ word (ὁ ∷ []) "John.1.10"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ ς ∷ []) "John.1.10"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.1.10"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.1.10"
∷ word (ἔ ∷ γ ∷ ν ∷ ω ∷ []) "John.1.10"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.1.11"
∷ word (τ ∷ ὰ ∷ []) "John.1.11"
∷ word (ἴ ∷ δ ∷ ι ∷ α ∷ []) "John.1.11"
∷ word (ἦ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.1.11"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.11"
∷ word (ο ∷ ἱ ∷ []) "John.1.11"
∷ word (ἴ ∷ δ ∷ ι ∷ ο ∷ ι ∷ []) "John.1.11"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.1.11"
∷ word (ο ∷ ὐ ∷ []) "John.1.11"
∷ word (π ∷ α ∷ ρ ∷ έ ∷ ∙λ ∷ α ∷ β ∷ ο ∷ ν ∷ []) "John.1.11"
∷ word (ὅ ∷ σ ∷ ο ∷ ι ∷ []) "John.1.12"
∷ word (δ ∷ ὲ ∷ []) "John.1.12"
∷ word (ἔ ∷ ∙λ ∷ α ∷ β ∷ ο ∷ ν ∷ []) "John.1.12"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.1.12"
∷ word (ἔ ∷ δ ∷ ω ∷ κ ∷ ε ∷ ν ∷ []) "John.1.12"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.1.12"
∷ word (ἐ ∷ ξ ∷ ο ∷ υ ∷ σ ∷ ί ∷ α ∷ ν ∷ []) "John.1.12"
∷ word (τ ∷ έ ∷ κ ∷ ν ∷ α ∷ []) "John.1.12"
∷ word (θ ∷ ε ∷ ο ∷ ῦ ∷ []) "John.1.12"
∷ word (γ ∷ ε ∷ ν ∷ έ ∷ σ ∷ θ ∷ α ∷ ι ∷ []) "John.1.12"
∷ word (τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.1.12"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ ο ∷ υ ∷ σ ∷ ι ∷ ν ∷ []) "John.1.12"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.1.12"
∷ word (τ ∷ ὸ ∷ []) "John.1.12"
∷ word (ὄ ∷ ν ∷ ο ∷ μ ∷ α ∷ []) "John.1.12"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.1.12"
∷ word (ο ∷ ἳ ∷ []) "John.1.13"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.1.13"
∷ word (ἐ ∷ ξ ∷ []) "John.1.13"
∷ word (α ∷ ἱ ∷ μ ∷ ά ∷ τ ∷ ω ∷ ν ∷ []) "John.1.13"
∷ word (ο ∷ ὐ ∷ δ ∷ ὲ ∷ []) "John.1.13"
∷ word (ἐ ∷ κ ∷ []) "John.1.13"
∷ word (θ ∷ ε ∷ ∙λ ∷ ή ∷ μ ∷ α ∷ τ ∷ ο ∷ ς ∷ []) "John.1.13"
∷ word (σ ∷ α ∷ ρ ∷ κ ∷ ὸ ∷ ς ∷ []) "John.1.13"
∷ word (ο ∷ ὐ ∷ δ ∷ ὲ ∷ []) "John.1.13"
∷ word (ἐ ∷ κ ∷ []) "John.1.13"
∷ word (θ ∷ ε ∷ ∙λ ∷ ή ∷ μ ∷ α ∷ τ ∷ ο ∷ ς ∷ []) "John.1.13"
∷ word (ἀ ∷ ν ∷ δ ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.1.13"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ []) "John.1.13"
∷ word (ἐ ∷ κ ∷ []) "John.1.13"
∷ word (θ ∷ ε ∷ ο ∷ ῦ ∷ []) "John.1.13"
∷ word (ἐ ∷ γ ∷ ε ∷ ν ∷ ν ∷ ή ∷ θ ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.1.13"
∷ word (Κ ∷ α ∷ ὶ ∷ []) "John.1.14"
∷ word (ὁ ∷ []) "John.1.14"
∷ word (∙λ ∷ ό ∷ γ ∷ ο ∷ ς ∷ []) "John.1.14"
∷ word (σ ∷ ὰ ∷ ρ ∷ ξ ∷ []) "John.1.14"
∷ word (ἐ ∷ γ ∷ έ ∷ ν ∷ ε ∷ τ ∷ ο ∷ []) "John.1.14"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.14"
∷ word (ἐ ∷ σ ∷ κ ∷ ή ∷ ν ∷ ω ∷ σ ∷ ε ∷ ν ∷ []) "John.1.14"
∷ word (ἐ ∷ ν ∷ []) "John.1.14"
∷ word (ἡ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.1.14"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.14"
∷ word (ἐ ∷ θ ∷ ε ∷ α ∷ σ ∷ ά ∷ μ ∷ ε ∷ θ ∷ α ∷ []) "John.1.14"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.1.14"
∷ word (δ ∷ ό ∷ ξ ∷ α ∷ ν ∷ []) "John.1.14"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.1.14"
∷ word (δ ∷ ό ∷ ξ ∷ α ∷ ν ∷ []) "John.1.14"
∷ word (ὡ ∷ ς ∷ []) "John.1.14"
∷ word (μ ∷ ο ∷ ν ∷ ο ∷ γ ∷ ε ∷ ν ∷ ο ∷ ῦ ∷ ς ∷ []) "John.1.14"
∷ word (π ∷ α ∷ ρ ∷ ὰ ∷ []) "John.1.14"
∷ word (π ∷ α ∷ τ ∷ ρ ∷ ό ∷ ς ∷ []) "John.1.14"
∷ word (π ∷ ∙λ ∷ ή ∷ ρ ∷ η ∷ ς ∷ []) "John.1.14"
∷ word (χ ∷ ά ∷ ρ ∷ ι ∷ τ ∷ ο ∷ ς ∷ []) "John.1.14"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.14"
∷ word (ἀ ∷ ∙λ ∷ η ∷ θ ∷ ε ∷ ί ∷ α ∷ ς ∷ []) "John.1.14"
∷ word (Ἰ ∷ ω ∷ ά ∷ ν ∷ ν ∷ η ∷ ς ∷ []) "John.1.15"
∷ word (μ ∷ α ∷ ρ ∷ τ ∷ υ ∷ ρ ∷ ε ∷ ῖ ∷ []) "John.1.15"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.1.15"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.1.15"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.15"
∷ word (κ ∷ έ ∷ κ ∷ ρ ∷ α ∷ γ ∷ ε ∷ ν ∷ []) "John.1.15"
∷ word (∙λ ∷ έ ∷ γ ∷ ω ∷ ν ∷ []) "John.1.15"
∷ word (Ο ∷ ὗ ∷ τ ∷ ο ∷ ς ∷ []) "John.1.15"
∷ word (ἦ ∷ ν ∷ []) "John.1.15"
∷ word (ὃ ∷ ν ∷ []) "John.1.15"
∷ word (ε ∷ ἶ ∷ π ∷ ο ∷ ν ∷ []) "John.1.15"
∷ word (Ὁ ∷ []) "John.1.15"
∷ word (ὀ ∷ π ∷ ί ∷ σ ∷ ω ∷ []) "John.1.15"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.1.15"
∷ word (ἐ ∷ ρ ∷ χ ∷ ό ∷ μ ∷ ε ∷ ν ∷ ο ∷ ς ∷ []) "John.1.15"
∷ word (ἔ ∷ μ ∷ π ∷ ρ ∷ ο ∷ σ ∷ θ ∷ έ ∷ ν ∷ []) "John.1.15"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.1.15"
∷ word (γ ∷ έ ∷ γ ∷ ο ∷ ν ∷ ε ∷ ν ∷ []) "John.1.15"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.1.15"
∷ word (π ∷ ρ ∷ ῶ ∷ τ ∷ ό ∷ ς ∷ []) "John.1.15"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.1.15"
∷ word (ἦ ∷ ν ∷ []) "John.1.15"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.1.16"
∷ word (ἐ ∷ κ ∷ []) "John.1.16"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.1.16"
∷ word (π ∷ ∙λ ∷ η ∷ ρ ∷ ώ ∷ μ ∷ α ∷ τ ∷ ο ∷ ς ∷ []) "John.1.16"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.1.16"
∷ word (ἡ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.1.16"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.1.16"
∷ word (ἐ ∷ ∙λ ∷ ά ∷ β ∷ ο ∷ μ ∷ ε ∷ ν ∷ []) "John.1.16"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.16"
∷ word (χ ∷ ά ∷ ρ ∷ ι ∷ ν ∷ []) "John.1.16"
∷ word (ἀ ∷ ν ∷ τ ∷ ὶ ∷ []) "John.1.16"
∷ word (χ ∷ ά ∷ ρ ∷ ι ∷ τ ∷ ο ∷ ς ∷ []) "John.1.16"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.1.17"
∷ word (ὁ ∷ []) "John.1.17"
∷ word (ν ∷ ό ∷ μ ∷ ο ∷ ς ∷ []) "John.1.17"
∷ word (δ ∷ ι ∷ ὰ ∷ []) "John.1.17"
∷ word (Μ ∷ ω ∷ ϋ ∷ σ ∷ έ ∷ ω ∷ ς ∷ []) "John.1.17"
∷ word (ἐ ∷ δ ∷ ό ∷ θ ∷ η ∷ []) "John.1.17"
∷ word (ἡ ∷ []) "John.1.17"
∷ word (χ ∷ ά ∷ ρ ∷ ι ∷ ς ∷ []) "John.1.17"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.17"
∷ word (ἡ ∷ []) "John.1.17"
∷ word (ἀ ∷ ∙λ ∷ ή ∷ θ ∷ ε ∷ ι ∷ α ∷ []) "John.1.17"
∷ word (δ ∷ ι ∷ ὰ ∷ []) "John.1.17"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ []) "John.1.17"
∷ word (Χ ∷ ρ ∷ ι ∷ σ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.1.17"
∷ word (ἐ ∷ γ ∷ έ ∷ ν ∷ ε ∷ τ ∷ ο ∷ []) "John.1.17"
∷ word (θ ∷ ε ∷ ὸ ∷ ν ∷ []) "John.1.18"
∷ word (ο ∷ ὐ ∷ δ ∷ ε ∷ ὶ ∷ ς ∷ []) "John.1.18"
∷ word (ἑ ∷ ώ ∷ ρ ∷ α ∷ κ ∷ ε ∷ ν ∷ []) "John.1.18"
∷ word (π ∷ ώ ∷ π ∷ ο ∷ τ ∷ ε ∷ []) "John.1.18"
∷ word (μ ∷ ο ∷ ν ∷ ο ∷ γ ∷ ε ∷ ν ∷ ὴ ∷ ς ∷ []) "John.1.18"
∷ word (θ ∷ ε ∷ ὸ ∷ ς ∷ []) "John.1.18"
∷ word (ὁ ∷ []) "John.1.18"
∷ word (ὢ ∷ ν ∷ []) "John.1.18"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.1.18"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.1.18"
∷ word (κ ∷ ό ∷ ∙λ ∷ π ∷ ο ∷ ν ∷ []) "John.1.18"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.1.18"
∷ word (π ∷ α ∷ τ ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.1.18"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ο ∷ ς ∷ []) "John.1.18"
∷ word (ἐ ∷ ξ ∷ η ∷ γ ∷ ή ∷ σ ∷ α ∷ τ ∷ ο ∷ []) "John.1.18"
∷ word (Κ ∷ α ∷ ὶ ∷ []) "John.1.19"
∷ word (α ∷ ὕ ∷ τ ∷ η ∷ []) "John.1.19"
∷ word (ἐ ∷ σ ∷ τ ∷ ὶ ∷ ν ∷ []) "John.1.19"
∷ word (ἡ ∷ []) "John.1.19"
∷ word (μ ∷ α ∷ ρ ∷ τ ∷ υ ∷ ρ ∷ ί ∷ α ∷ []) "John.1.19"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.1.19"
∷ word (Ἰ ∷ ω ∷ ά ∷ ν ∷ ν ∷ ο ∷ υ ∷ []) "John.1.19"
∷ word (ὅ ∷ τ ∷ ε ∷ []) "John.1.19"
∷ word (ἀ ∷ π ∷ έ ∷ σ ∷ τ ∷ ε ∷ ι ∷ ∙λ ∷ α ∷ ν ∷ []) "John.1.19"
∷ word (ο ∷ ἱ ∷ []) "John.1.19"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ῖ ∷ ο ∷ ι ∷ []) "John.1.19"
∷ word (ἐ ∷ ξ ∷ []) "John.1.19"
∷ word (Ἱ ∷ ε ∷ ρ ∷ ο ∷ σ ∷ ο ∷ ∙λ ∷ ύ ∷ μ ∷ ω ∷ ν ∷ []) "John.1.19"
∷ word (ἱ ∷ ε ∷ ρ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.1.19"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.19"
∷ word (Λ ∷ ε ∷ υ ∷ ί ∷ τ ∷ α ∷ ς ∷ []) "John.1.19"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.1.19"
∷ word (ἐ ∷ ρ ∷ ω ∷ τ ∷ ή ∷ σ ∷ ω ∷ σ ∷ ι ∷ ν ∷ []) "John.1.19"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.1.19"
∷ word (Σ ∷ ὺ ∷ []) "John.1.19"
∷ word (τ ∷ ί ∷ ς ∷ []) "John.1.19"
∷ word (ε ∷ ἶ ∷ []) "John.1.19"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.20"
∷ word (ὡ ∷ μ ∷ ο ∷ ∙λ ∷ ό ∷ γ ∷ η ∷ σ ∷ ε ∷ ν ∷ []) "John.1.20"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.20"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.1.20"
∷ word (ἠ ∷ ρ ∷ ν ∷ ή ∷ σ ∷ α ∷ τ ∷ ο ∷ []) "John.1.20"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.20"
∷ word (ὡ ∷ μ ∷ ο ∷ ∙λ ∷ ό ∷ γ ∷ η ∷ σ ∷ ε ∷ ν ∷ []) "John.1.20"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.1.20"
∷ word (Ἐ ∷ γ ∷ ὼ ∷ []) "John.1.20"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.1.20"
∷ word (ε ∷ ἰ ∷ μ ∷ ὶ ∷ []) "John.1.20"
∷ word (ὁ ∷ []) "John.1.20"
∷ word (χ ∷ ρ ∷ ι ∷ σ ∷ τ ∷ ό ∷ ς ∷ []) "John.1.20"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.21"
∷ word (ἠ ∷ ρ ∷ ώ ∷ τ ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.1.21"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.1.21"
∷ word (Τ ∷ ί ∷ []) "John.1.21"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.1.21"
∷ word (σ ∷ ὺ ∷ []) "John.1.21"
∷ word (Ἠ ∷ ∙λ ∷ ί ∷ α ∷ ς ∷ []) "John.1.21"
∷ word (ε ∷ ἶ ∷ []) "John.1.21"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.21"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.1.21"
∷ word (Ο ∷ ὐ ∷ κ ∷ []) "John.1.21"
∷ word (ε ∷ ἰ ∷ μ ∷ ί ∷ []) "John.1.21"
∷ word (Ὁ ∷ []) "John.1.21"
∷ word (π ∷ ρ ∷ ο ∷ φ ∷ ή ∷ τ ∷ η ∷ ς ∷ []) "John.1.21"
∷ word (ε ∷ ἶ ∷ []) "John.1.21"
∷ word (σ ∷ ύ ∷ []) "John.1.21"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.21"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.1.21"
∷ word (Ο ∷ ὔ ∷ []) "John.1.21"
∷ word (ε ∷ ἶ ∷ π ∷ α ∷ ν ∷ []) "John.1.22"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.1.22"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.1.22"
∷ word (Τ ∷ ί ∷ ς ∷ []) "John.1.22"
∷ word (ε ∷ ἶ ∷ []) "John.1.22"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.1.22"
∷ word (ἀ ∷ π ∷ ό ∷ κ ∷ ρ ∷ ι ∷ σ ∷ ι ∷ ν ∷ []) "John.1.22"
∷ word (δ ∷ ῶ ∷ μ ∷ ε ∷ ν ∷ []) "John.1.22"
∷ word (τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.1.22"
∷ word (π ∷ έ ∷ μ ∷ ψ ∷ α ∷ σ ∷ ι ∷ ν ∷ []) "John.1.22"
∷ word (ἡ ∷ μ ∷ ᾶ ∷ ς ∷ []) "John.1.22"
∷ word (τ ∷ ί ∷ []) "John.1.22"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ ς ∷ []) "John.1.22"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.1.22"
∷ word (σ ∷ ε ∷ α ∷ υ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.1.22"
∷ word (ἔ ∷ φ ∷ η ∷ []) "John.1.23"
∷ word (Ἐ ∷ γ ∷ ὼ ∷ []) "John.1.23"
∷ word (φ ∷ ω ∷ ν ∷ ὴ ∷ []) "John.1.23"
∷ word (β ∷ ο ∷ ῶ ∷ ν ∷ τ ∷ ο ∷ ς ∷ []) "John.1.23"
∷ word (ἐ ∷ ν ∷ []) "John.1.23"
∷ word (τ ∷ ῇ ∷ []) "John.1.23"
∷ word (ἐ ∷ ρ ∷ ή ∷ μ ∷ ῳ ∷ []) "John.1.23"
∷ word (Ε ∷ ὐ ∷ θ ∷ ύ ∷ ν ∷ α ∷ τ ∷ ε ∷ []) "John.1.23"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.1.23"
∷ word (ὁ ∷ δ ∷ ὸ ∷ ν ∷ []) "John.1.23"
∷ word (κ ∷ υ ∷ ρ ∷ ί ∷ ο ∷ υ ∷ []) "John.1.23"
∷ word (κ ∷ α ∷ θ ∷ ὼ ∷ ς ∷ []) "John.1.23"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.1.23"
∷ word (Ἠ ∷ σ ∷ α ∷ ΐ ∷ α ∷ ς ∷ []) "John.1.23"
∷ word (ὁ ∷ []) "John.1.23"
∷ word (π ∷ ρ ∷ ο ∷ φ ∷ ή ∷ τ ∷ η ∷ ς ∷ []) "John.1.23"
∷ word (Κ ∷ α ∷ ὶ ∷ []) "John.1.24"
∷ word (ἀ ∷ π ∷ ε ∷ σ ∷ τ ∷ α ∷ ∙λ ∷ μ ∷ έ ∷ ν ∷ ο ∷ ι ∷ []) "John.1.24"
∷ word (ἦ ∷ σ ∷ α ∷ ν ∷ []) "John.1.24"
∷ word (ἐ ∷ κ ∷ []) "John.1.24"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.1.24"
∷ word (Φ ∷ α ∷ ρ ∷ ι ∷ σ ∷ α ∷ ί ∷ ω ∷ ν ∷ []) "John.1.24"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.25"
∷ word (ἠ ∷ ρ ∷ ώ ∷ τ ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.1.25"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.1.25"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.25"
∷ word (ε ∷ ἶ ∷ π ∷ α ∷ ν ∷ []) "John.1.25"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.1.25"
∷ word (Τ ∷ ί ∷ []) "John.1.25"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.1.25"
∷ word (β ∷ α ∷ π ∷ τ ∷ ί ∷ ζ ∷ ε ∷ ι ∷ ς ∷ []) "John.1.25"
∷ word (ε ∷ ἰ ∷ []) "John.1.25"
∷ word (σ ∷ ὺ ∷ []) "John.1.25"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.1.25"
∷ word (ε ∷ ἶ ∷ []) "John.1.25"
∷ word (ὁ ∷ []) "John.1.25"
∷ word (χ ∷ ρ ∷ ι ∷ σ ∷ τ ∷ ὸ ∷ ς ∷ []) "John.1.25"
∷ word (ο ∷ ὐ ∷ δ ∷ ὲ ∷ []) "John.1.25"
∷ word (Ἠ ∷ ∙λ ∷ ί ∷ α ∷ ς ∷ []) "John.1.25"
∷ word (ο ∷ ὐ ∷ δ ∷ ὲ ∷ []) "John.1.25"
∷ word (ὁ ∷ []) "John.1.25"
∷ word (π ∷ ρ ∷ ο ∷ φ ∷ ή ∷ τ ∷ η ∷ ς ∷ []) "John.1.25"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.1.26"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.1.26"
∷ word (ὁ ∷ []) "John.1.26"
∷ word (Ἰ ∷ ω ∷ ά ∷ ν ∷ ν ∷ η ∷ ς ∷ []) "John.1.26"
∷ word (∙λ ∷ έ ∷ γ ∷ ω ∷ ν ∷ []) "John.1.26"
∷ word (Ἐ ∷ γ ∷ ὼ ∷ []) "John.1.26"
∷ word (β ∷ α ∷ π ∷ τ ∷ ί ∷ ζ ∷ ω ∷ []) "John.1.26"
∷ word (ἐ ∷ ν ∷ []) "John.1.26"
∷ word (ὕ ∷ δ ∷ α ∷ τ ∷ ι ∷ []) "John.1.26"
∷ word (μ ∷ έ ∷ σ ∷ ο ∷ ς ∷ []) "John.1.26"
∷ word (ὑ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.1.26"
∷ word (ἕ ∷ σ ∷ τ ∷ η ∷ κ ∷ ε ∷ ν ∷ []) "John.1.26"
∷ word (ὃ ∷ ν ∷ []) "John.1.26"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.1.26"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.1.26"
∷ word (ο ∷ ἴ ∷ δ ∷ α ∷ τ ∷ ε ∷ []) "John.1.26"
∷ word (ὁ ∷ []) "John.1.27"
∷ word (ὀ ∷ π ∷ ί ∷ σ ∷ ω ∷ []) "John.1.27"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.1.27"
∷ word (ἐ ∷ ρ ∷ χ ∷ ό ∷ μ ∷ ε ∷ ν ∷ ο ∷ ς ∷ []) "John.1.27"
∷ word (ο ∷ ὗ ∷ []) "John.1.27"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.1.27"
∷ word (ε ∷ ἰ ∷ μ ∷ ὶ ∷ []) "John.1.27"
∷ word (ἄ ∷ ξ ∷ ι ∷ ο ∷ ς ∷ []) "John.1.27"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.1.27"
∷ word (∙λ ∷ ύ ∷ σ ∷ ω ∷ []) "John.1.27"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.1.27"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.1.27"
∷ word (ἱ ∷ μ ∷ ά ∷ ν ∷ τ ∷ α ∷ []) "John.1.27"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.1.27"
∷ word (ὑ ∷ π ∷ ο ∷ δ ∷ ή ∷ μ ∷ α ∷ τ ∷ ο ∷ ς ∷ []) "John.1.27"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.1.28"
∷ word (ἐ ∷ ν ∷ []) "John.1.28"
∷ word (Β ∷ η ∷ θ ∷ α ∷ ν ∷ ί ∷ ᾳ ∷ []) "John.1.28"
∷ word (ἐ ∷ γ ∷ έ ∷ ν ∷ ε ∷ τ ∷ ο ∷ []) "John.1.28"
∷ word (π ∷ έ ∷ ρ ∷ α ∷ ν ∷ []) "John.1.28"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.1.28"
∷ word (Ἰ ∷ ο ∷ ρ ∷ δ ∷ ά ∷ ν ∷ ο ∷ υ ∷ []) "John.1.28"
∷ word (ὅ ∷ π ∷ ο ∷ υ ∷ []) "John.1.28"
∷ word (ἦ ∷ ν ∷ []) "John.1.28"
∷ word (ὁ ∷ []) "John.1.28"
∷ word (Ἰ ∷ ω ∷ ά ∷ ν ∷ ν ∷ η ∷ ς ∷ []) "John.1.28"
∷ word (β ∷ α ∷ π ∷ τ ∷ ί ∷ ζ ∷ ω ∷ ν ∷ []) "John.1.28"
∷ word (Τ ∷ ῇ ∷ []) "John.1.29"
∷ word (ἐ ∷ π ∷ α ∷ ύ ∷ ρ ∷ ι ∷ ο ∷ ν ∷ []) "John.1.29"
∷ word (β ∷ ∙λ ∷ έ ∷ π ∷ ε ∷ ι ∷ []) "John.1.29"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.1.29"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ν ∷ []) "John.1.29"
∷ word (ἐ ∷ ρ ∷ χ ∷ ό ∷ μ ∷ ε ∷ ν ∷ ο ∷ ν ∷ []) "John.1.29"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.1.29"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.1.29"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.29"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.1.29"
∷ word (Ἴ ∷ δ ∷ ε ∷ []) "John.1.29"
∷ word (ὁ ∷ []) "John.1.29"
∷ word (ἀ ∷ μ ∷ ν ∷ ὸ ∷ ς ∷ []) "John.1.29"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.1.29"
∷ word (θ ∷ ε ∷ ο ∷ ῦ ∷ []) "John.1.29"
∷ word (ὁ ∷ []) "John.1.29"
∷ word (α ∷ ἴ ∷ ρ ∷ ω ∷ ν ∷ []) "John.1.29"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.1.29"
∷ word (ἁ ∷ μ ∷ α ∷ ρ ∷ τ ∷ ί ∷ α ∷ ν ∷ []) "John.1.29"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.1.29"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ υ ∷ []) "John.1.29"
∷ word (ο ∷ ὗ ∷ τ ∷ ό ∷ ς ∷ []) "John.1.30"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.1.30"
∷ word (ὑ ∷ π ∷ ὲ ∷ ρ ∷ []) "John.1.30"
∷ word (ο ∷ ὗ ∷ []) "John.1.30"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.1.30"
∷ word (ε ∷ ἶ ∷ π ∷ ο ∷ ν ∷ []) "John.1.30"
∷ word (Ὀ ∷ π ∷ ί ∷ σ ∷ ω ∷ []) "John.1.30"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.1.30"
∷ word (ἔ ∷ ρ ∷ χ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.1.30"
∷ word (ἀ ∷ ν ∷ ὴ ∷ ρ ∷ []) "John.1.30"
∷ word (ὃ ∷ ς ∷ []) "John.1.30"
∷ word (ἔ ∷ μ ∷ π ∷ ρ ∷ ο ∷ σ ∷ θ ∷ έ ∷ ν ∷ []) "John.1.30"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.1.30"
∷ word (γ ∷ έ ∷ γ ∷ ο ∷ ν ∷ ε ∷ ν ∷ []) "John.1.30"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.1.30"
∷ word (π ∷ ρ ∷ ῶ ∷ τ ∷ ό ∷ ς ∷ []) "John.1.30"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.1.30"
∷ word (ἦ ∷ ν ∷ []) "John.1.30"
∷ word (κ ∷ ἀ ∷ γ ∷ ὼ ∷ []) "John.1.31"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.1.31"
∷ word (ᾔ ∷ δ ∷ ε ∷ ι ∷ ν ∷ []) "John.1.31"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.1.31"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ []) "John.1.31"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.1.31"
∷ word (φ ∷ α ∷ ν ∷ ε ∷ ρ ∷ ω ∷ θ ∷ ῇ ∷ []) "John.1.31"
∷ word (τ ∷ ῷ ∷ []) "John.1.31"
∷ word (Ἰ ∷ σ ∷ ρ ∷ α ∷ ὴ ∷ ∙λ ∷ []) "John.1.31"
∷ word (δ ∷ ι ∷ ὰ ∷ []) "John.1.31"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.1.31"
∷ word (ἦ ∷ ∙λ ∷ θ ∷ ο ∷ ν ∷ []) "John.1.31"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.1.31"
∷ word (ἐ ∷ ν ∷ []) "John.1.31"
∷ word (ὕ ∷ δ ∷ α ∷ τ ∷ ι ∷ []) "John.1.31"
∷ word (β ∷ α ∷ π ∷ τ ∷ ί ∷ ζ ∷ ω ∷ ν ∷ []) "John.1.31"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.32"
∷ word (ἐ ∷ μ ∷ α ∷ ρ ∷ τ ∷ ύ ∷ ρ ∷ η ∷ σ ∷ ε ∷ ν ∷ []) "John.1.32"
∷ word (Ἰ ∷ ω ∷ ά ∷ ν ∷ ν ∷ η ∷ ς ∷ []) "John.1.32"
∷ word (∙λ ∷ έ ∷ γ ∷ ω ∷ ν ∷ []) "John.1.32"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.1.32"
∷ word (Τ ∷ ε ∷ θ ∷ έ ∷ α ∷ μ ∷ α ∷ ι ∷ []) "John.1.32"
∷ word (τ ∷ ὸ ∷ []) "John.1.32"
∷ word (π ∷ ν ∷ ε ∷ ῦ ∷ μ ∷ α ∷ []) "John.1.32"
∷ word (κ ∷ α ∷ τ ∷ α ∷ β ∷ α ∷ ῖ ∷ ν ∷ ο ∷ ν ∷ []) "John.1.32"
∷ word (ὡ ∷ ς ∷ []) "John.1.32"
∷ word (π ∷ ε ∷ ρ ∷ ι ∷ σ ∷ τ ∷ ε ∷ ρ ∷ ὰ ∷ ν ∷ []) "John.1.32"
∷ word (ἐ ∷ ξ ∷ []) "John.1.32"
∷ word (ο ∷ ὐ ∷ ρ ∷ α ∷ ν ∷ ο ∷ ῦ ∷ []) "John.1.32"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.32"
∷ word (ἔ ∷ μ ∷ ε ∷ ι ∷ ν ∷ ε ∷ ν ∷ []) "John.1.32"
∷ word (ἐ ∷ π ∷ []) "John.1.32"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.1.32"
∷ word (κ ∷ ἀ ∷ γ ∷ ὼ ∷ []) "John.1.33"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.1.33"
∷ word (ᾔ ∷ δ ∷ ε ∷ ι ∷ ν ∷ []) "John.1.33"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.1.33"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ []) "John.1.33"
∷ word (ὁ ∷ []) "John.1.33"
∷ word (π ∷ έ ∷ μ ∷ ψ ∷ α ∷ ς ∷ []) "John.1.33"
∷ word (μ ∷ ε ∷ []) "John.1.33"
∷ word (β ∷ α ∷ π ∷ τ ∷ ί ∷ ζ ∷ ε ∷ ι ∷ ν ∷ []) "John.1.33"
∷ word (ἐ ∷ ν ∷ []) "John.1.33"
∷ word (ὕ ∷ δ ∷ α ∷ τ ∷ ι ∷ []) "John.1.33"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ό ∷ ς ∷ []) "John.1.33"
∷ word (μ ∷ ο ∷ ι ∷ []) "John.1.33"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.1.33"
∷ word (Ἐ ∷ φ ∷ []) "John.1.33"
∷ word (ὃ ∷ ν ∷ []) "John.1.33"
∷ word (ἂ ∷ ν ∷ []) "John.1.33"
∷ word (ἴ ∷ δ ∷ ῃ ∷ ς ∷ []) "John.1.33"
∷ word (τ ∷ ὸ ∷ []) "John.1.33"
∷ word (π ∷ ν ∷ ε ∷ ῦ ∷ μ ∷ α ∷ []) "John.1.33"
∷ word (κ ∷ α ∷ τ ∷ α ∷ β ∷ α ∷ ῖ ∷ ν ∷ ο ∷ ν ∷ []) "John.1.33"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.33"
∷ word (μ ∷ έ ∷ ν ∷ ο ∷ ν ∷ []) "John.1.33"
∷ word (ἐ ∷ π ∷ []) "John.1.33"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.1.33"
∷ word (ο ∷ ὗ ∷ τ ∷ ό ∷ ς ∷ []) "John.1.33"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.1.33"
∷ word (ὁ ∷ []) "John.1.33"
∷ word (β ∷ α ∷ π ∷ τ ∷ ί ∷ ζ ∷ ω ∷ ν ∷ []) "John.1.33"
∷ word (ἐ ∷ ν ∷ []) "John.1.33"
∷ word (π ∷ ν ∷ ε ∷ ύ ∷ μ ∷ α ∷ τ ∷ ι ∷ []) "John.1.33"
∷ word (ἁ ∷ γ ∷ ί ∷ ῳ ∷ []) "John.1.33"
∷ word (κ ∷ ἀ ∷ γ ∷ ὼ ∷ []) "John.1.34"
∷ word (ἑ ∷ ώ ∷ ρ ∷ α ∷ κ ∷ α ∷ []) "John.1.34"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.34"
∷ word (μ ∷ ε ∷ μ ∷ α ∷ ρ ∷ τ ∷ ύ ∷ ρ ∷ η ∷ κ ∷ α ∷ []) "John.1.34"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.1.34"
∷ word (ο ∷ ὗ ∷ τ ∷ ό ∷ ς ∷ []) "John.1.34"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.1.34"
∷ word (ὁ ∷ []) "John.1.34"
∷ word (ἐ ∷ κ ∷ ∙λ ∷ ε ∷ κ ∷ τ ∷ ὸ ∷ ς ∷ []) "John.1.34"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.1.34"
∷ word (θ ∷ ε ∷ ο ∷ ῦ ∷ []) "John.1.34"
∷ word (Τ ∷ ῇ ∷ []) "John.1.35"
∷ word (ἐ ∷ π ∷ α ∷ ύ ∷ ρ ∷ ι ∷ ο ∷ ν ∷ []) "John.1.35"
∷ word (π ∷ ά ∷ ∙λ ∷ ι ∷ ν ∷ []) "John.1.35"
∷ word (ε ∷ ἱ ∷ σ ∷ τ ∷ ή ∷ κ ∷ ε ∷ ι ∷ []) "John.1.35"
∷ word (ὁ ∷ []) "John.1.35"
∷ word (Ἰ ∷ ω ∷ ά ∷ ν ∷ ν ∷ η ∷ ς ∷ []) "John.1.35"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.35"
∷ word (ἐ ∷ κ ∷ []) "John.1.35"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.1.35"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ ῶ ∷ ν ∷ []) "John.1.35"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.1.35"
∷ word (δ ∷ ύ ∷ ο ∷ []) "John.1.35"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.36"
∷ word (ἐ ∷ μ ∷ β ∷ ∙λ ∷ έ ∷ ψ ∷ α ∷ ς ∷ []) "John.1.36"
∷ word (τ ∷ ῷ ∷ []) "John.1.36"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ []) "John.1.36"
∷ word (π ∷ ε ∷ ρ ∷ ι ∷ π ∷ α ∷ τ ∷ ο ∷ ῦ ∷ ν ∷ τ ∷ ι ∷ []) "John.1.36"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.1.36"
∷ word (Ἴ ∷ δ ∷ ε ∷ []) "John.1.36"
∷ word (ὁ ∷ []) "John.1.36"
∷ word (ἀ ∷ μ ∷ ν ∷ ὸ ∷ ς ∷ []) "John.1.36"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.1.36"
∷ word (θ ∷ ε ∷ ο ∷ ῦ ∷ []) "John.1.36"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.37"
∷ word (ἤ ∷ κ ∷ ο ∷ υ ∷ σ ∷ α ∷ ν ∷ []) "John.1.37"
∷ word (ο ∷ ἱ ∷ []) "John.1.37"
∷ word (δ ∷ ύ ∷ ο ∷ []) "John.1.37"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ α ∷ ὶ ∷ []) "John.1.37"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.1.37"
∷ word (∙λ ∷ α ∷ ∙λ ∷ ο ∷ ῦ ∷ ν ∷ τ ∷ ο ∷ ς ∷ []) "John.1.37"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.37"
∷ word (ἠ ∷ κ ∷ ο ∷ ∙λ ∷ ο ∷ ύ ∷ θ ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.1.37"
∷ word (τ ∷ ῷ ∷ []) "John.1.37"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ []) "John.1.37"
∷ word (σ ∷ τ ∷ ρ ∷ α ∷ φ ∷ ε ∷ ὶ ∷ ς ∷ []) "John.1.38"
∷ word (δ ∷ ὲ ∷ []) "John.1.38"
∷ word (ὁ ∷ []) "John.1.38"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.1.38"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.38"
∷ word (θ ∷ ε ∷ α ∷ σ ∷ ά ∷ μ ∷ ε ∷ ν ∷ ο ∷ ς ∷ []) "John.1.38"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.1.38"
∷ word (ἀ ∷ κ ∷ ο ∷ ∙λ ∷ ο ∷ υ ∷ θ ∷ ο ∷ ῦ ∷ ν ∷ τ ∷ α ∷ ς ∷ []) "John.1.38"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.1.38"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.1.38"
∷ word (Τ ∷ ί ∷ []) "John.1.38"
∷ word (ζ ∷ η ∷ τ ∷ ε ∷ ῖ ∷ τ ∷ ε ∷ []) "John.1.38"
∷ word (ο ∷ ἱ ∷ []) "John.1.38"
∷ word (δ ∷ ὲ ∷ []) "John.1.38"
∷ word (ε ∷ ἶ ∷ π ∷ α ∷ ν ∷ []) "John.1.38"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.1.38"
∷ word (Ῥ ∷ α ∷ β ∷ β ∷ ί ∷ []) "John.1.38"
∷ word (ὃ ∷ []) "John.1.38"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.1.38"
∷ word (μ ∷ ε ∷ θ ∷ ε ∷ ρ ∷ μ ∷ η ∷ ν ∷ ε ∷ υ ∷ ό ∷ μ ∷ ε ∷ ν ∷ ο ∷ ν ∷ []) "John.1.38"
∷ word (Δ ∷ ι ∷ δ ∷ ά ∷ σ ∷ κ ∷ α ∷ ∙λ ∷ ε ∷ []) "John.1.38"
∷ word (π ∷ ο ∷ ῦ ∷ []) "John.1.38"
∷ word (μ ∷ έ ∷ ν ∷ ε ∷ ι ∷ ς ∷ []) "John.1.38"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.1.39"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.1.39"
∷ word (Ἔ ∷ ρ ∷ χ ∷ ε ∷ σ ∷ θ ∷ ε ∷ []) "John.1.39"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.39"
∷ word (ὄ ∷ ψ ∷ ε ∷ σ ∷ θ ∷ ε ∷ []) "John.1.39"
∷ word (ἦ ∷ ∙λ ∷ θ ∷ α ∷ ν ∷ []) "John.1.39"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.1.39"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.39"
∷ word (ε ∷ ἶ ∷ δ ∷ α ∷ ν ∷ []) "John.1.39"
∷ word (π ∷ ο ∷ ῦ ∷ []) "John.1.39"
∷ word (μ ∷ έ ∷ ν ∷ ε ∷ ι ∷ []) "John.1.39"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.39"
∷ word (π ∷ α ∷ ρ ∷ []) "John.1.39"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.1.39"
∷ word (ἔ ∷ μ ∷ ε ∷ ι ∷ ν ∷ α ∷ ν ∷ []) "John.1.39"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.1.39"
∷ word (ἡ ∷ μ ∷ έ ∷ ρ ∷ α ∷ ν ∷ []) "John.1.39"
∷ word (ἐ ∷ κ ∷ ε ∷ ί ∷ ν ∷ η ∷ ν ∷ []) "John.1.39"
∷ word (ὥ ∷ ρ ∷ α ∷ []) "John.1.39"
∷ word (ἦ ∷ ν ∷ []) "John.1.39"
∷ word (ὡ ∷ ς ∷ []) "John.1.39"
∷ word (δ ∷ ε ∷ κ ∷ ά ∷ τ ∷ η ∷ []) "John.1.39"
∷ word (ἦ ∷ ν ∷ []) "John.1.40"
∷ word (Ἀ ∷ ν ∷ δ ∷ ρ ∷ έ ∷ α ∷ ς ∷ []) "John.1.40"
∷ word (ὁ ∷ []) "John.1.40"
∷ word (ἀ ∷ δ ∷ ε ∷ ∙λ ∷ φ ∷ ὸ ∷ ς ∷ []) "John.1.40"
∷ word (Σ ∷ ί ∷ μ ∷ ω ∷ ν ∷ ο ∷ ς ∷ []) "John.1.40"
∷ word (Π ∷ έ ∷ τ ∷ ρ ∷ ο ∷ υ ∷ []) "John.1.40"
∷ word (ε ∷ ἷ ∷ ς ∷ []) "John.1.40"
∷ word (ἐ ∷ κ ∷ []) "John.1.40"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.1.40"
∷ word (δ ∷ ύ ∷ ο ∷ []) "John.1.40"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.1.40"
∷ word (ἀ ∷ κ ∷ ο ∷ υ ∷ σ ∷ ά ∷ ν ∷ τ ∷ ω ∷ ν ∷ []) "John.1.40"
∷ word (π ∷ α ∷ ρ ∷ ὰ ∷ []) "John.1.40"
∷ word (Ἰ ∷ ω ∷ ά ∷ ν ∷ ν ∷ ο ∷ υ ∷ []) "John.1.40"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.40"
∷ word (ἀ ∷ κ ∷ ο ∷ ∙λ ∷ ο ∷ υ ∷ θ ∷ η ∷ σ ∷ ά ∷ ν ∷ τ ∷ ω ∷ ν ∷ []) "John.1.40"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.1.40"
∷ word (ε ∷ ὑ ∷ ρ ∷ ί ∷ σ ∷ κ ∷ ε ∷ ι ∷ []) "John.1.41"
∷ word (ο ∷ ὗ ∷ τ ∷ ο ∷ ς ∷ []) "John.1.41"
∷ word (π ∷ ρ ∷ ῶ ∷ τ ∷ ο ∷ ν ∷ []) "John.1.41"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.1.41"
∷ word (ἀ ∷ δ ∷ ε ∷ ∙λ ∷ φ ∷ ὸ ∷ ν ∷ []) "John.1.41"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.1.41"
∷ word (ἴ ∷ δ ∷ ι ∷ ο ∷ ν ∷ []) "John.1.41"
∷ word (Σ ∷ ί ∷ μ ∷ ω ∷ ν ∷ α ∷ []) "John.1.41"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.41"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.1.41"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.1.41"
∷ word (Ε ∷ ὑ ∷ ρ ∷ ή ∷ κ ∷ α ∷ μ ∷ ε ∷ ν ∷ []) "John.1.41"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.1.41"
∷ word (Μ ∷ ε ∷ σ ∷ σ ∷ ί ∷ α ∷ ν ∷ []) "John.1.41"
∷ word (ὅ ∷ []) "John.1.41"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.1.41"
∷ word (μ ∷ ε ∷ θ ∷ ε ∷ ρ ∷ μ ∷ η ∷ ν ∷ ε ∷ υ ∷ ό ∷ μ ∷ ε ∷ ν ∷ ο ∷ ν ∷ []) "John.1.41"
∷ word (χ ∷ ρ ∷ ι ∷ σ ∷ τ ∷ ό ∷ ς ∷ []) "John.1.41"
∷ word (ἤ ∷ γ ∷ α ∷ γ ∷ ε ∷ ν ∷ []) "John.1.42"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.1.42"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.1.42"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.1.42"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ν ∷ []) "John.1.42"
∷ word (ἐ ∷ μ ∷ β ∷ ∙λ ∷ έ ∷ ψ ∷ α ∷ ς ∷ []) "John.1.42"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.1.42"
∷ word (ὁ ∷ []) "John.1.42"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.1.42"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.1.42"
∷ word (Σ ∷ ὺ ∷ []) "John.1.42"
∷ word (ε ∷ ἶ ∷ []) "John.1.42"
∷ word (Σ ∷ ί ∷ μ ∷ ω ∷ ν ∷ []) "John.1.42"
∷ word (ὁ ∷ []) "John.1.42"
∷ word (υ ∷ ἱ ∷ ὸ ∷ ς ∷ []) "John.1.42"
∷ word (Ἰ ∷ ω ∷ ά ∷ ν ∷ ν ∷ ο ∷ υ ∷ []) "John.1.42"
∷ word (σ ∷ ὺ ∷ []) "John.1.42"
∷ word (κ ∷ ∙λ ∷ η ∷ θ ∷ ή ∷ σ ∷ ῃ ∷ []) "John.1.42"
∷ word (Κ ∷ η ∷ φ ∷ ᾶ ∷ ς ∷ []) "John.1.42"
∷ word (ὃ ∷ []) "John.1.42"
∷ word (ἑ ∷ ρ ∷ μ ∷ η ∷ ν ∷ ε ∷ ύ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.1.42"
∷ word (Π ∷ έ ∷ τ ∷ ρ ∷ ο ∷ ς ∷ []) "John.1.42"
∷ word (Τ ∷ ῇ ∷ []) "John.1.43"
∷ word (ἐ ∷ π ∷ α ∷ ύ ∷ ρ ∷ ι ∷ ο ∷ ν ∷ []) "John.1.43"
∷ word (ἠ ∷ θ ∷ έ ∷ ∙λ ∷ η ∷ σ ∷ ε ∷ ν ∷ []) "John.1.43"
∷ word (ἐ ∷ ξ ∷ ε ∷ ∙λ ∷ θ ∷ ε ∷ ῖ ∷ ν ∷ []) "John.1.43"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.1.43"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.1.43"
∷ word (Γ ∷ α ∷ ∙λ ∷ ι ∷ ∙λ ∷ α ∷ ί ∷ α ∷ ν ∷ []) "John.1.43"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.43"
∷ word (ε ∷ ὑ ∷ ρ ∷ ί ∷ σ ∷ κ ∷ ε ∷ ι ∷ []) "John.1.43"
∷ word (Φ ∷ ί ∷ ∙λ ∷ ι ∷ π ∷ π ∷ ο ∷ ν ∷ []) "John.1.43"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.43"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.1.43"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.1.43"
∷ word (ὁ ∷ []) "John.1.43"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.1.43"
∷ word (Ἀ ∷ κ ∷ ο ∷ ∙λ ∷ ο ∷ ύ ∷ θ ∷ ε ∷ ι ∷ []) "John.1.43"
∷ word (μ ∷ ο ∷ ι ∷ []) "John.1.43"
∷ word (ἦ ∷ ν ∷ []) "John.1.44"
∷ word (δ ∷ ὲ ∷ []) "John.1.44"
∷ word (ὁ ∷ []) "John.1.44"
∷ word (Φ ∷ ί ∷ ∙λ ∷ ι ∷ π ∷ π ∷ ο ∷ ς ∷ []) "John.1.44"
∷ word (ἀ ∷ π ∷ ὸ ∷ []) "John.1.44"
∷ word (Β ∷ η ∷ θ ∷ σ ∷ α ∷ ϊ ∷ δ ∷ ά ∷ []) "John.1.44"
∷ word (ἐ ∷ κ ∷ []) "John.1.44"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.1.44"
∷ word (π ∷ ό ∷ ∙λ ∷ ε ∷ ω ∷ ς ∷ []) "John.1.44"
∷ word (Ἀ ∷ ν ∷ δ ∷ ρ ∷ έ ∷ ο ∷ υ ∷ []) "John.1.44"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.44"
∷ word (Π ∷ έ ∷ τ ∷ ρ ∷ ο ∷ υ ∷ []) "John.1.44"
∷ word (ε ∷ ὑ ∷ ρ ∷ ί ∷ σ ∷ κ ∷ ε ∷ ι ∷ []) "John.1.45"
∷ word (Φ ∷ ί ∷ ∙λ ∷ ι ∷ π ∷ π ∷ ο ∷ ς ∷ []) "John.1.45"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.1.45"
∷ word (Ν ∷ α ∷ θ ∷ α ∷ ν ∷ α ∷ ὴ ∷ ∙λ ∷ []) "John.1.45"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.45"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.1.45"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.1.45"
∷ word (Ὃ ∷ ν ∷ []) "John.1.45"
∷ word (ἔ ∷ γ ∷ ρ ∷ α ∷ ψ ∷ ε ∷ ν ∷ []) "John.1.45"
∷ word (Μ ∷ ω ∷ ϋ ∷ σ ∷ ῆ ∷ ς ∷ []) "John.1.45"
∷ word (ἐ ∷ ν ∷ []) "John.1.45"
∷ word (τ ∷ ῷ ∷ []) "John.1.45"
∷ word (ν ∷ ό ∷ μ ∷ ῳ ∷ []) "John.1.45"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.45"
∷ word (ο ∷ ἱ ∷ []) "John.1.45"
∷ word (π ∷ ρ ∷ ο ∷ φ ∷ ῆ ∷ τ ∷ α ∷ ι ∷ []) "John.1.45"
∷ word (ε ∷ ὑ ∷ ρ ∷ ή ∷ κ ∷ α ∷ μ ∷ ε ∷ ν ∷ []) "John.1.45"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ν ∷ []) "John.1.45"
∷ word (υ ∷ ἱ ∷ ὸ ∷ ν ∷ []) "John.1.45"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.1.45"
∷ word (Ἰ ∷ ω ∷ σ ∷ ὴ ∷ φ ∷ []) "John.1.45"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.1.45"
∷ word (ἀ ∷ π ∷ ὸ ∷ []) "John.1.45"
∷ word (Ν ∷ α ∷ ζ ∷ α ∷ ρ ∷ έ ∷ τ ∷ []) "John.1.45"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.46"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.1.46"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.1.46"
∷ word (Ν ∷ α ∷ θ ∷ α ∷ ν ∷ α ∷ ή ∷ ∙λ ∷ []) "John.1.46"
∷ word (Ἐ ∷ κ ∷ []) "John.1.46"
∷ word (Ν ∷ α ∷ ζ ∷ α ∷ ρ ∷ ὲ ∷ τ ∷ []) "John.1.46"
∷ word (δ ∷ ύ ∷ ν ∷ α ∷ τ ∷ α ∷ ί ∷ []) "John.1.46"
∷ word (τ ∷ ι ∷ []) "John.1.46"
∷ word (ἀ ∷ γ ∷ α ∷ θ ∷ ὸ ∷ ν ∷ []) "John.1.46"
∷ word (ε ∷ ἶ ∷ ν ∷ α ∷ ι ∷ []) "John.1.46"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.1.46"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.1.46"
∷ word (ὁ ∷ []) "John.1.46"
∷ word (Φ ∷ ί ∷ ∙λ ∷ ι ∷ π ∷ π ∷ ο ∷ ς ∷ []) "John.1.46"
∷ word (Ἔ ∷ ρ ∷ χ ∷ ο ∷ υ ∷ []) "John.1.46"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.46"
∷ word (ἴ ∷ δ ∷ ε ∷ []) "John.1.46"
∷ word (ε ∷ ἶ ∷ δ ∷ ε ∷ ν ∷ []) "John.1.47"
∷ word (ὁ ∷ []) "John.1.47"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.1.47"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.1.47"
∷ word (Ν ∷ α ∷ θ ∷ α ∷ ν ∷ α ∷ ὴ ∷ ∙λ ∷ []) "John.1.47"
∷ word (ἐ ∷ ρ ∷ χ ∷ ό ∷ μ ∷ ε ∷ ν ∷ ο ∷ ν ∷ []) "John.1.47"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.1.47"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.1.47"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.47"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.1.47"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.1.47"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.1.47"
∷ word (Ἴ ∷ δ ∷ ε ∷ []) "John.1.47"
∷ word (ἀ ∷ ∙λ ∷ η ∷ θ ∷ ῶ ∷ ς ∷ []) "John.1.47"
∷ word (Ἰ ∷ σ ∷ ρ ∷ α ∷ η ∷ ∙λ ∷ ί ∷ τ ∷ η ∷ ς ∷ []) "John.1.47"
∷ word (ἐ ∷ ν ∷ []) "John.1.47"
∷ word (ᾧ ∷ []) "John.1.47"
∷ word (δ ∷ ό ∷ ∙λ ∷ ο ∷ ς ∷ []) "John.1.47"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.1.47"
∷ word (ἔ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.1.47"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.1.48"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.1.48"
∷ word (Ν ∷ α ∷ θ ∷ α ∷ ν ∷ α ∷ ή ∷ ∙λ ∷ []) "John.1.48"
∷ word (Π ∷ ό ∷ θ ∷ ε ∷ ν ∷ []) "John.1.48"
∷ word (μ ∷ ε ∷ []) "John.1.48"
∷ word (γ ∷ ι ∷ ν ∷ ώ ∷ σ ∷ κ ∷ ε ∷ ι ∷ ς ∷ []) "John.1.48"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.1.48"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.1.48"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.48"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.1.48"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.1.48"
∷ word (Π ∷ ρ ∷ ὸ ∷ []) "John.1.48"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.1.48"
∷ word (σ ∷ ε ∷ []) "John.1.48"
∷ word (Φ ∷ ί ∷ ∙λ ∷ ι ∷ π ∷ π ∷ ο ∷ ν ∷ []) "John.1.48"
∷ word (φ ∷ ω ∷ ν ∷ ῆ ∷ σ ∷ α ∷ ι ∷ []) "John.1.48"
∷ word (ὄ ∷ ν ∷ τ ∷ α ∷ []) "John.1.48"
∷ word (ὑ ∷ π ∷ ὸ ∷ []) "John.1.48"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.1.48"
∷ word (σ ∷ υ ∷ κ ∷ ῆ ∷ ν ∷ []) "John.1.48"
∷ word (ε ∷ ἶ ∷ δ ∷ ό ∷ ν ∷ []) "John.1.48"
∷ word (σ ∷ ε ∷ []) "John.1.48"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.1.49"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.1.49"
∷ word (Ν ∷ α ∷ θ ∷ α ∷ ν ∷ α ∷ ή ∷ ∙λ ∷ []) "John.1.49"
∷ word (Ῥ ∷ α ∷ β ∷ β ∷ ί ∷ []) "John.1.49"
∷ word (σ ∷ ὺ ∷ []) "John.1.49"
∷ word (ε ∷ ἶ ∷ []) "John.1.49"
∷ word (ὁ ∷ []) "John.1.49"
∷ word (υ ∷ ἱ ∷ ὸ ∷ ς ∷ []) "John.1.49"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.1.49"
∷ word (θ ∷ ε ∷ ο ∷ ῦ ∷ []) "John.1.49"
∷ word (σ ∷ ὺ ∷ []) "John.1.49"
∷ word (β ∷ α ∷ σ ∷ ι ∷ ∙λ ∷ ε ∷ ὺ ∷ ς ∷ []) "John.1.49"
∷ word (ε ∷ ἶ ∷ []) "John.1.49"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.1.49"
∷ word (Ἰ ∷ σ ∷ ρ ∷ α ∷ ή ∷ ∙λ ∷ []) "John.1.49"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.1.50"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.1.50"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.50"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.1.50"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.1.50"
∷ word (Ὅ ∷ τ ∷ ι ∷ []) "John.1.50"
∷ word (ε ∷ ἶ ∷ π ∷ ό ∷ ν ∷ []) "John.1.50"
∷ word (σ ∷ ο ∷ ι ∷ []) "John.1.50"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.1.50"
∷ word (ε ∷ ἶ ∷ δ ∷ ό ∷ ν ∷ []) "John.1.50"
∷ word (σ ∷ ε ∷ []) "John.1.50"
∷ word (ὑ ∷ π ∷ ο ∷ κ ∷ ά ∷ τ ∷ ω ∷ []) "John.1.50"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.1.50"
∷ word (σ ∷ υ ∷ κ ∷ ῆ ∷ ς ∷ []) "John.1.50"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ ε ∷ ι ∷ ς ∷ []) "John.1.50"
∷ word (μ ∷ ε ∷ ί ∷ ζ ∷ ω ∷ []) "John.1.50"
∷ word (τ ∷ ο ∷ ύ ∷ τ ∷ ω ∷ ν ∷ []) "John.1.50"
∷ word (ὄ ∷ ψ ∷ ῃ ∷ []) "John.1.50"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.51"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.1.51"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.1.51"
∷ word (Ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.1.51"
∷ word (ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.1.51"
∷ word (∙λ ∷ έ ∷ γ ∷ ω ∷ []) "John.1.51"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.1.51"
∷ word (ὄ ∷ ψ ∷ ε ∷ σ ∷ θ ∷ ε ∷ []) "John.1.51"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.1.51"
∷ word (ο ∷ ὐ ∷ ρ ∷ α ∷ ν ∷ ὸ ∷ ν ∷ []) "John.1.51"
∷ word (ἀ ∷ ν ∷ ε ∷ ῳ ∷ γ ∷ ό ∷ τ ∷ α ∷ []) "John.1.51"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.51"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.1.51"
∷ word (ἀ ∷ γ ∷ γ ∷ έ ∷ ∙λ ∷ ο ∷ υ ∷ ς ∷ []) "John.1.51"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.1.51"
∷ word (θ ∷ ε ∷ ο ∷ ῦ ∷ []) "John.1.51"
∷ word (ἀ ∷ ν ∷ α ∷ β ∷ α ∷ ί ∷ ν ∷ ο ∷ ν ∷ τ ∷ α ∷ ς ∷ []) "John.1.51"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.1.51"
∷ word (κ ∷ α ∷ τ ∷ α ∷ β ∷ α ∷ ί ∷ ν ∷ ο ∷ ν ∷ τ ∷ α ∷ ς ∷ []) "John.1.51"
∷ word (ἐ ∷ π ∷ ὶ ∷ []) "John.1.51"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.1.51"
∷ word (υ ∷ ἱ ∷ ὸ ∷ ν ∷ []) "John.1.51"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.1.51"
∷ word (ἀ ∷ ν ∷ θ ∷ ρ ∷ ώ ∷ π ∷ ο ∷ υ ∷ []) "John.1.51"
∷ word (Κ ∷ α ∷ ὶ ∷ []) "John.2.1"
∷ word (τ ∷ ῇ ∷ []) "John.2.1"
∷ word (ἡ ∷ μ ∷ έ ∷ ρ ∷ ᾳ ∷ []) "John.2.1"
∷ word (τ ∷ ῇ ∷ []) "John.2.1"
∷ word (τ ∷ ρ ∷ ί ∷ τ ∷ ῃ ∷ []) "John.2.1"
∷ word (γ ∷ ά ∷ μ ∷ ο ∷ ς ∷ []) "John.2.1"
∷ word (ἐ ∷ γ ∷ έ ∷ ν ∷ ε ∷ τ ∷ ο ∷ []) "John.2.1"
∷ word (ἐ ∷ ν ∷ []) "John.2.1"
∷ word (Κ ∷ α ∷ ν ∷ ὰ ∷ []) "John.2.1"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.2.1"
∷ word (Γ ∷ α ∷ ∙λ ∷ ι ∷ ∙λ ∷ α ∷ ί ∷ α ∷ ς ∷ []) "John.2.1"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.2.1"
∷ word (ἦ ∷ ν ∷ []) "John.2.1"
∷ word (ἡ ∷ []) "John.2.1"
∷ word (μ ∷ ή ∷ τ ∷ η ∷ ρ ∷ []) "John.2.1"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.2.1"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ []) "John.2.1"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ []) "John.2.1"
∷ word (ἐ ∷ κ ∷ ∙λ ∷ ή ∷ θ ∷ η ∷ []) "John.2.2"
∷ word (δ ∷ ὲ ∷ []) "John.2.2"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.2.2"
∷ word (ὁ ∷ []) "John.2.2"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.2.2"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.2.2"
∷ word (ο ∷ ἱ ∷ []) "John.2.2"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ α ∷ ὶ ∷ []) "John.2.2"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.2.2"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.2.2"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.2.2"
∷ word (γ ∷ ά ∷ μ ∷ ο ∷ ν ∷ []) "John.2.2"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.2.3"
∷ word (ὑ ∷ σ ∷ τ ∷ ε ∷ ρ ∷ ή ∷ σ ∷ α ∷ ν ∷ τ ∷ ο ∷ ς ∷ []) "John.2.3"
∷ word (ο ∷ ἴ ∷ ν ∷ ο ∷ υ ∷ []) "John.2.3"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.2.3"
∷ word (ἡ ∷ []) "John.2.3"
∷ word (μ ∷ ή ∷ τ ∷ η ∷ ρ ∷ []) "John.2.3"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.2.3"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ []) "John.2.3"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.2.3"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.2.3"
∷ word (Ο ∷ ἶ ∷ ν ∷ ο ∷ ν ∷ []) "John.2.3"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.2.3"
∷ word (ἔ ∷ χ ∷ ο ∷ υ ∷ σ ∷ ι ∷ ν ∷ []) "John.2.3"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.2.4"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.2.4"
∷ word (α ∷ ὐ ∷ τ ∷ ῇ ∷ []) "John.2.4"
∷ word (ὁ ∷ []) "John.2.4"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.2.4"
∷ word (Τ ∷ ί ∷ []) "John.2.4"
∷ word (ἐ ∷ μ ∷ ο ∷ ὶ ∷ []) "John.2.4"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.2.4"
∷ word (σ ∷ ο ∷ ί ∷ []) "John.2.4"
∷ word (γ ∷ ύ ∷ ν ∷ α ∷ ι ∷ []) "John.2.4"
∷ word (ο ∷ ὔ ∷ π ∷ ω ∷ []) "John.2.4"
∷ word (ἥ ∷ κ ∷ ε ∷ ι ∷ []) "John.2.4"
∷ word (ἡ ∷ []) "John.2.4"
∷ word (ὥ ∷ ρ ∷ α ∷ []) "John.2.4"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.2.4"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.2.5"
∷ word (ἡ ∷ []) "John.2.5"
∷ word (μ ∷ ή ∷ τ ∷ η ∷ ρ ∷ []) "John.2.5"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.2.5"
∷ word (τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.2.5"
∷ word (δ ∷ ι ∷ α ∷ κ ∷ ό ∷ ν ∷ ο ∷ ι ∷ ς ∷ []) "John.2.5"
∷ word (Ὅ ∷ []) "John.2.5"
∷ word (τ ∷ ι ∷ []) "John.2.5"
∷ word (ἂ ∷ ν ∷ []) "John.2.5"
∷ word (∙λ ∷ έ ∷ γ ∷ ῃ ∷ []) "John.2.5"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.2.5"
∷ word (π ∷ ο ∷ ι ∷ ή ∷ σ ∷ α ∷ τ ∷ ε ∷ []) "John.2.5"
∷ word (ἦ ∷ σ ∷ α ∷ ν ∷ []) "John.2.6"
∷ word (δ ∷ ὲ ∷ []) "John.2.6"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ []) "John.2.6"
∷ word (∙λ ∷ ί ∷ θ ∷ ι ∷ ν ∷ α ∷ ι ∷ []) "John.2.6"
∷ word (ὑ ∷ δ ∷ ρ ∷ ί ∷ α ∷ ι ∷ []) "John.2.6"
∷ word (ἓ ∷ ξ ∷ []) "John.2.6"
∷ word (κ ∷ α ∷ τ ∷ ὰ ∷ []) "John.2.6"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.2.6"
∷ word (κ ∷ α ∷ θ ∷ α ∷ ρ ∷ ι ∷ σ ∷ μ ∷ ὸ ∷ ν ∷ []) "John.2.6"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.2.6"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ί ∷ ω ∷ ν ∷ []) "John.2.6"
∷ word (κ ∷ ε ∷ ί ∷ μ ∷ ε ∷ ν ∷ α ∷ ι ∷ []) "John.2.6"
∷ word (χ ∷ ω ∷ ρ ∷ ο ∷ ῦ ∷ σ ∷ α ∷ ι ∷ []) "John.2.6"
∷ word (ἀ ∷ ν ∷ ὰ ∷ []) "John.2.6"
∷ word (μ ∷ ε ∷ τ ∷ ρ ∷ η ∷ τ ∷ ὰ ∷ ς ∷ []) "John.2.6"
∷ word (δ ∷ ύ ∷ ο ∷ []) "John.2.6"
∷ word (ἢ ∷ []) "John.2.6"
∷ word (τ ∷ ρ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.2.6"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.2.7"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.2.7"
∷ word (ὁ ∷ []) "John.2.7"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.2.7"
∷ word (Γ ∷ ε ∷ μ ∷ ί ∷ σ ∷ α ∷ τ ∷ ε ∷ []) "John.2.7"
∷ word (τ ∷ ὰ ∷ ς ∷ []) "John.2.7"
∷ word (ὑ ∷ δ ∷ ρ ∷ ί ∷ α ∷ ς ∷ []) "John.2.7"
∷ word (ὕ ∷ δ ∷ α ∷ τ ∷ ο ∷ ς ∷ []) "John.2.7"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.2.7"
∷ word (ἐ ∷ γ ∷ έ ∷ μ ∷ ι ∷ σ ∷ α ∷ ν ∷ []) "John.2.7"
∷ word (α ∷ ὐ ∷ τ ∷ ὰ ∷ ς ∷ []) "John.2.7"
∷ word (ἕ ∷ ω ∷ ς ∷ []) "John.2.7"
∷ word (ἄ ∷ ν ∷ ω ∷ []) "John.2.7"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.2.8"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.2.8"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.2.8"
∷ word (Ἀ ∷ ν ∷ τ ∷ ∙λ ∷ ή ∷ σ ∷ α ∷ τ ∷ ε ∷ []) "John.2.8"
∷ word (ν ∷ ῦ ∷ ν ∷ []) "John.2.8"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.2.8"
∷ word (φ ∷ έ ∷ ρ ∷ ε ∷ τ ∷ ε ∷ []) "John.2.8"
∷ word (τ ∷ ῷ ∷ []) "John.2.8"
∷ word (ἀ ∷ ρ ∷ χ ∷ ι ∷ τ ∷ ρ ∷ ι ∷ κ ∷ ∙λ ∷ ί ∷ ν ∷ ῳ ∷ []) "John.2.8"
∷ word (ο ∷ ἱ ∷ []) "John.2.8"
∷ word (δ ∷ ὲ ∷ []) "John.2.8"
∷ word (ἤ ∷ ν ∷ ε ∷ γ ∷ κ ∷ α ∷ ν ∷ []) "John.2.8"
∷ word (ὡ ∷ ς ∷ []) "John.2.9"
∷ word (δ ∷ ὲ ∷ []) "John.2.9"
∷ word (ἐ ∷ γ ∷ ε ∷ ύ ∷ σ ∷ α ∷ τ ∷ ο ∷ []) "John.2.9"
∷ word (ὁ ∷ []) "John.2.9"
∷ word (ἀ ∷ ρ ∷ χ ∷ ι ∷ τ ∷ ρ ∷ ί ∷ κ ∷ ∙λ ∷ ι ∷ ν ∷ ο ∷ ς ∷ []) "John.2.9"
∷ word (τ ∷ ὸ ∷ []) "John.2.9"
∷ word (ὕ ∷ δ ∷ ω ∷ ρ ∷ []) "John.2.9"
∷ word (ο ∷ ἶ ∷ ν ∷ ο ∷ ν ∷ []) "John.2.9"
∷ word (γ ∷ ε ∷ γ ∷ ε ∷ ν ∷ η ∷ μ ∷ έ ∷ ν ∷ ο ∷ ν ∷ []) "John.2.9"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.2.9"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.2.9"
∷ word (ᾔ ∷ δ ∷ ε ∷ ι ∷ []) "John.2.9"
∷ word (π ∷ ό ∷ θ ∷ ε ∷ ν ∷ []) "John.2.9"
∷ word (ἐ ∷ σ ∷ τ ∷ ί ∷ ν ∷ []) "John.2.9"
∷ word (ο ∷ ἱ ∷ []) "John.2.9"
∷ word (δ ∷ ὲ ∷ []) "John.2.9"
∷ word (δ ∷ ι ∷ ά ∷ κ ∷ ο ∷ ν ∷ ο ∷ ι ∷ []) "John.2.9"
∷ word (ᾔ ∷ δ ∷ ε ∷ ι ∷ σ ∷ α ∷ ν ∷ []) "John.2.9"
∷ word (ο ∷ ἱ ∷ []) "John.2.9"
∷ word (ἠ ∷ ν ∷ τ ∷ ∙λ ∷ η ∷ κ ∷ ό ∷ τ ∷ ε ∷ ς ∷ []) "John.2.9"
∷ word (τ ∷ ὸ ∷ []) "John.2.9"
∷ word (ὕ ∷ δ ∷ ω ∷ ρ ∷ []) "John.2.9"
∷ word (φ ∷ ω ∷ ν ∷ ε ∷ ῖ ∷ []) "John.2.9"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.2.9"
∷ word (ν ∷ υ ∷ μ ∷ φ ∷ ί ∷ ο ∷ ν ∷ []) "John.2.9"
∷ word (ὁ ∷ []) "John.2.9"
∷ word (ἀ ∷ ρ ∷ χ ∷ ι ∷ τ ∷ ρ ∷ ί ∷ κ ∷ ∙λ ∷ ι ∷ ν ∷ ο ∷ ς ∷ []) "John.2.9"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.2.10"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.2.10"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.2.10"
∷ word (Π ∷ ᾶ ∷ ς ∷ []) "John.2.10"
∷ word (ἄ ∷ ν ∷ θ ∷ ρ ∷ ω ∷ π ∷ ο ∷ ς ∷ []) "John.2.10"
∷ word (π ∷ ρ ∷ ῶ ∷ τ ∷ ο ∷ ν ∷ []) "John.2.10"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.2.10"
∷ word (κ ∷ α ∷ ∙λ ∷ ὸ ∷ ν ∷ []) "John.2.10"
∷ word (ο ∷ ἶ ∷ ν ∷ ο ∷ ν ∷ []) "John.2.10"
∷ word (τ ∷ ί ∷ θ ∷ η ∷ σ ∷ ι ∷ ν ∷ []) "John.2.10"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.2.10"
∷ word (ὅ ∷ τ ∷ α ∷ ν ∷ []) "John.2.10"
∷ word (μ ∷ ε ∷ θ ∷ υ ∷ σ ∷ θ ∷ ῶ ∷ σ ∷ ι ∷ ν ∷ []) "John.2.10"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.2.10"
∷ word (ἐ ∷ ∙λ ∷ ά ∷ σ ∷ σ ∷ ω ∷ []) "John.2.10"
∷ word (σ ∷ ὺ ∷ []) "John.2.10"
∷ word (τ ∷ ε ∷ τ ∷ ή ∷ ρ ∷ η ∷ κ ∷ α ∷ ς ∷ []) "John.2.10"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.2.10"
∷ word (κ ∷ α ∷ ∙λ ∷ ὸ ∷ ν ∷ []) "John.2.10"
∷ word (ο ∷ ἶ ∷ ν ∷ ο ∷ ν ∷ []) "John.2.10"
∷ word (ἕ ∷ ω ∷ ς ∷ []) "John.2.10"
∷ word (ἄ ∷ ρ ∷ τ ∷ ι ∷ []) "John.2.10"
∷ word (τ ∷ α ∷ ύ ∷ τ ∷ η ∷ ν ∷ []) "John.2.11"
∷ word (ἐ ∷ π ∷ ο ∷ ί ∷ η ∷ σ ∷ ε ∷ ν ∷ []) "John.2.11"
∷ word (ἀ ∷ ρ ∷ χ ∷ ὴ ∷ ν ∷ []) "John.2.11"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.2.11"
∷ word (σ ∷ η ∷ μ ∷ ε ∷ ί ∷ ω ∷ ν ∷ []) "John.2.11"
∷ word (ὁ ∷ []) "John.2.11"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.2.11"
∷ word (ἐ ∷ ν ∷ []) "John.2.11"
∷ word (Κ ∷ α ∷ ν ∷ ὰ ∷ []) "John.2.11"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.2.11"
∷ word (Γ ∷ α ∷ ∙λ ∷ ι ∷ ∙λ ∷ α ∷ ί ∷ α ∷ ς ∷ []) "John.2.11"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.2.11"
∷ word (ἐ ∷ φ ∷ α ∷ ν ∷ έ ∷ ρ ∷ ω ∷ σ ∷ ε ∷ ν ∷ []) "John.2.11"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.2.11"
∷ word (δ ∷ ό ∷ ξ ∷ α ∷ ν ∷ []) "John.2.11"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.2.11"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.2.11"
∷ word (ἐ ∷ π ∷ ί ∷ σ ∷ τ ∷ ε ∷ υ ∷ σ ∷ α ∷ ν ∷ []) "John.2.11"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.2.11"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.2.11"
∷ word (ο ∷ ἱ ∷ []) "John.2.11"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ α ∷ ὶ ∷ []) "John.2.11"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.2.11"
∷ word (Μ ∷ ε ∷ τ ∷ ὰ ∷ []) "John.2.12"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.2.12"
∷ word (κ ∷ α ∷ τ ∷ έ ∷ β ∷ η ∷ []) "John.2.12"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.2.12"
∷ word (Κ ∷ α ∷ φ ∷ α ∷ ρ ∷ ν ∷ α ∷ ο ∷ ὺ ∷ μ ∷ []) "John.2.12"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ς ∷ []) "John.2.12"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.2.12"
∷ word (ἡ ∷ []) "John.2.12"
∷ word (μ ∷ ή ∷ τ ∷ η ∷ ρ ∷ []) "John.2.12"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.2.12"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.2.12"
∷ word (ο ∷ ἱ ∷ []) "John.2.12"
∷ word (ἀ ∷ δ ∷ ε ∷ ∙λ ∷ φ ∷ ο ∷ ὶ ∷ []) "John.2.12"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.2.12"
∷ word (ο ∷ ἱ ∷ []) "John.2.12"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ α ∷ ὶ ∷ []) "John.2.12"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.2.12"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.2.12"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ []) "John.2.12"
∷ word (ἔ ∷ μ ∷ ε ∷ ι ∷ ν ∷ α ∷ ν ∷ []) "John.2.12"
∷ word (ο ∷ ὐ ∷ []) "John.2.12"
∷ word (π ∷ ο ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ ς ∷ []) "John.2.12"
∷ word (ἡ ∷ μ ∷ έ ∷ ρ ∷ α ∷ ς ∷ []) "John.2.12"
∷ word (Κ ∷ α ∷ ὶ ∷ []) "John.2.13"
∷ word (ἐ ∷ γ ∷ γ ∷ ὺ ∷ ς ∷ []) "John.2.13"
∷ word (ἦ ∷ ν ∷ []) "John.2.13"
∷ word (τ ∷ ὸ ∷ []) "John.2.13"
∷ word (π ∷ ά ∷ σ ∷ χ ∷ α ∷ []) "John.2.13"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.2.13"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ί ∷ ω ∷ ν ∷ []) "John.2.13"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.2.13"
∷ word (ἀ ∷ ν ∷ έ ∷ β ∷ η ∷ []) "John.2.13"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.2.13"
∷ word (Ἱ ∷ ε ∷ ρ ∷ ο ∷ σ ∷ ό ∷ ∙λ ∷ υ ∷ μ ∷ α ∷ []) "John.2.13"
∷ word (ὁ ∷ []) "John.2.13"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.2.13"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.2.14"
∷ word (ε ∷ ὗ ∷ ρ ∷ ε ∷ ν ∷ []) "John.2.14"
∷ word (ἐ ∷ ν ∷ []) "John.2.14"
∷ word (τ ∷ ῷ ∷ []) "John.2.14"
∷ word (ἱ ∷ ε ∷ ρ ∷ ῷ ∷ []) "John.2.14"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.2.14"
∷ word (π ∷ ω ∷ ∙λ ∷ ο ∷ ῦ ∷ ν ∷ τ ∷ α ∷ ς ∷ []) "John.2.14"
∷ word (β ∷ ό ∷ α ∷ ς ∷ []) "John.2.14"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.2.14"
∷ word (π ∷ ρ ∷ ό ∷ β ∷ α ∷ τ ∷ α ∷ []) "John.2.14"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.2.14"
∷ word (π ∷ ε ∷ ρ ∷ ι ∷ σ ∷ τ ∷ ε ∷ ρ ∷ ὰ ∷ ς ∷ []) "John.2.14"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.2.14"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.2.14"
∷ word (κ ∷ ε ∷ ρ ∷ μ ∷ α ∷ τ ∷ ι ∷ σ ∷ τ ∷ ὰ ∷ ς ∷ []) "John.2.14"
∷ word (κ ∷ α ∷ θ ∷ η ∷ μ ∷ έ ∷ ν ∷ ο ∷ υ ∷ ς ∷ []) "John.2.14"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.2.15"
∷ word (π ∷ ο ∷ ι ∷ ή ∷ σ ∷ α ∷ ς ∷ []) "John.2.15"
∷ word (φ ∷ ρ ∷ α ∷ γ ∷ έ ∷ ∙λ ∷ ∙λ ∷ ι ∷ ο ∷ ν ∷ []) "John.2.15"
∷ word (ἐ ∷ κ ∷ []) "John.2.15"
∷ word (σ ∷ χ ∷ ο ∷ ι ∷ ν ∷ ί ∷ ω ∷ ν ∷ []) "John.2.15"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ α ∷ ς ∷ []) "John.2.15"
∷ word (ἐ ∷ ξ ∷ έ ∷ β ∷ α ∷ ∙λ ∷ ε ∷ ν ∷ []) "John.2.15"
∷ word (ἐ ∷ κ ∷ []) "John.2.15"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.2.15"
∷ word (ἱ ∷ ε ∷ ρ ∷ ο ∷ ῦ ∷ []) "John.2.15"
∷ word (τ ∷ ά ∷ []) "John.2.15"
∷ word (τ ∷ ε ∷ []) "John.2.15"
∷ word (π ∷ ρ ∷ ό ∷ β ∷ α ∷ τ ∷ α ∷ []) "John.2.15"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.2.15"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.2.15"
∷ word (β ∷ ό ∷ α ∷ ς ∷ []) "John.2.15"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.2.15"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.2.15"
∷ word (κ ∷ ο ∷ ∙λ ∷ ∙λ ∷ υ ∷ β ∷ ι ∷ σ ∷ τ ∷ ῶ ∷ ν ∷ []) "John.2.15"
∷ word (ἐ ∷ ξ ∷ έ ∷ χ ∷ ε ∷ ε ∷ ν ∷ []) "John.2.15"
∷ word (τ ∷ ὰ ∷ []) "John.2.15"
∷ word (κ ∷ έ ∷ ρ ∷ μ ∷ α ∷ τ ∷ α ∷ []) "John.2.15"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.2.15"
∷ word (τ ∷ ὰ ∷ ς ∷ []) "John.2.15"
∷ word (τ ∷ ρ ∷ α ∷ π ∷ έ ∷ ζ ∷ α ∷ ς ∷ []) "John.2.15"
∷ word (ἀ ∷ ν ∷ έ ∷ σ ∷ τ ∷ ρ ∷ ε ∷ ψ ∷ ε ∷ ν ∷ []) "John.2.15"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.2.16"
∷ word (τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.2.16"
∷ word (τ ∷ ὰ ∷ ς ∷ []) "John.2.16"
∷ word (π ∷ ε ∷ ρ ∷ ι ∷ σ ∷ τ ∷ ε ∷ ρ ∷ ὰ ∷ ς ∷ []) "John.2.16"
∷ word (π ∷ ω ∷ ∙λ ∷ ο ∷ ῦ ∷ σ ∷ ι ∷ ν ∷ []) "John.2.16"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.2.16"
∷ word (Ἄ ∷ ρ ∷ α ∷ τ ∷ ε ∷ []) "John.2.16"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.2.16"
∷ word (ἐ ∷ ν ∷ τ ∷ ε ∷ ῦ ∷ θ ∷ ε ∷ ν ∷ []) "John.2.16"
∷ word (μ ∷ ὴ ∷ []) "John.2.16"
∷ word (π ∷ ο ∷ ι ∷ ε ∷ ῖ ∷ τ ∷ ε ∷ []) "John.2.16"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.2.16"
∷ word (ο ∷ ἶ ∷ κ ∷ ο ∷ ν ∷ []) "John.2.16"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.2.16"
∷ word (π ∷ α ∷ τ ∷ ρ ∷ ό ∷ ς ∷ []) "John.2.16"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.2.16"
∷ word (ο ∷ ἶ ∷ κ ∷ ο ∷ ν ∷ []) "John.2.16"
∷ word (ἐ ∷ μ ∷ π ∷ ο ∷ ρ ∷ ί ∷ ο ∷ υ ∷ []) "John.2.16"
∷ word (ἐ ∷ μ ∷ ν ∷ ή ∷ σ ∷ θ ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.2.17"
∷ word (ο ∷ ἱ ∷ []) "John.2.17"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ α ∷ ὶ ∷ []) "John.2.17"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.2.17"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.2.17"
∷ word (γ ∷ ε ∷ γ ∷ ρ ∷ α ∷ μ ∷ μ ∷ έ ∷ ν ∷ ο ∷ ν ∷ []) "John.2.17"
∷ word (ἐ ∷ σ ∷ τ ∷ ί ∷ ν ∷ []) "John.2.17"
∷ word (Ὁ ∷ []) "John.2.17"
∷ word (ζ ∷ ῆ ∷ ∙λ ∷ ο ∷ ς ∷ []) "John.2.17"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.2.17"
∷ word (ο ∷ ἴ ∷ κ ∷ ο ∷ υ ∷ []) "John.2.17"
∷ word (σ ∷ ο ∷ υ ∷ []) "John.2.17"
∷ word (κ ∷ α ∷ τ ∷ α ∷ φ ∷ ά ∷ γ ∷ ε ∷ τ ∷ α ∷ ί ∷ []) "John.2.17"
∷ word (μ ∷ ε ∷ []) "John.2.17"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.2.18"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.2.18"
∷ word (ο ∷ ἱ ∷ []) "John.2.18"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ῖ ∷ ο ∷ ι ∷ []) "John.2.18"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.2.18"
∷ word (ε ∷ ἶ ∷ π ∷ α ∷ ν ∷ []) "John.2.18"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.2.18"
∷ word (Τ ∷ ί ∷ []) "John.2.18"
∷ word (σ ∷ η ∷ μ ∷ ε ∷ ῖ ∷ ο ∷ ν ∷ []) "John.2.18"
∷ word (δ ∷ ε ∷ ι ∷ κ ∷ ν ∷ ύ ∷ ε ∷ ι ∷ ς ∷ []) "John.2.18"
∷ word (ἡ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.2.18"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.2.18"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.2.18"
∷ word (π ∷ ο ∷ ι ∷ ε ∷ ῖ ∷ ς ∷ []) "John.2.18"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.2.19"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.2.19"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.2.19"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.2.19"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.2.19"
∷ word (Λ ∷ ύ ∷ σ ∷ α ∷ τ ∷ ε ∷ []) "John.2.19"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.2.19"
∷ word (ν ∷ α ∷ ὸ ∷ ν ∷ []) "John.2.19"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ ν ∷ []) "John.2.19"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.2.19"
∷ word (ἐ ∷ ν ∷ []) "John.2.19"
∷ word (τ ∷ ρ ∷ ι ∷ σ ∷ ὶ ∷ ν ∷ []) "John.2.19"
∷ word (ἡ ∷ μ ∷ έ ∷ ρ ∷ α ∷ ι ∷ ς ∷ []) "John.2.19"
∷ word (ἐ ∷ γ ∷ ε ∷ ρ ∷ ῶ ∷ []) "John.2.19"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.2.19"
∷ word (ε ∷ ἶ ∷ π ∷ α ∷ ν ∷ []) "John.2.20"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.2.20"
∷ word (ο ∷ ἱ ∷ []) "John.2.20"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ῖ ∷ ο ∷ ι ∷ []) "John.2.20"
∷ word (Τ ∷ ε ∷ σ ∷ σ ∷ ε ∷ ρ ∷ ά ∷ κ ∷ ο ∷ ν ∷ τ ∷ α ∷ []) "John.2.20"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.2.20"
∷ word (ἓ ∷ ξ ∷ []) "John.2.20"
∷ word (ἔ ∷ τ ∷ ε ∷ σ ∷ ι ∷ ν ∷ []) "John.2.20"
∷ word (ο ∷ ἰ ∷ κ ∷ ο ∷ δ ∷ ο ∷ μ ∷ ή ∷ θ ∷ η ∷ []) "John.2.20"
∷ word (ὁ ∷ []) "John.2.20"
∷ word (ν ∷ α ∷ ὸ ∷ ς ∷ []) "John.2.20"
∷ word (ο ∷ ὗ ∷ τ ∷ ο ∷ ς ∷ []) "John.2.20"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.2.20"
∷ word (σ ∷ ὺ ∷ []) "John.2.20"
∷ word (ἐ ∷ ν ∷ []) "John.2.20"
∷ word (τ ∷ ρ ∷ ι ∷ σ ∷ ὶ ∷ ν ∷ []) "John.2.20"
∷ word (ἡ ∷ μ ∷ έ ∷ ρ ∷ α ∷ ι ∷ ς ∷ []) "John.2.20"
∷ word (ἐ ∷ γ ∷ ε ∷ ρ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.2.20"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.2.20"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ο ∷ ς ∷ []) "John.2.21"
∷ word (δ ∷ ὲ ∷ []) "John.2.21"
∷ word (ἔ ∷ ∙λ ∷ ε ∷ γ ∷ ε ∷ ν ∷ []) "John.2.21"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.2.21"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.2.21"
∷ word (ν ∷ α ∷ ο ∷ ῦ ∷ []) "John.2.21"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.2.21"
∷ word (σ ∷ ώ ∷ μ ∷ α ∷ τ ∷ ο ∷ ς ∷ []) "John.2.21"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.2.21"
∷ word (ὅ ∷ τ ∷ ε ∷ []) "John.2.22"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.2.22"
∷ word (ἠ ∷ γ ∷ έ ∷ ρ ∷ θ ∷ η ∷ []) "John.2.22"
∷ word (ἐ ∷ κ ∷ []) "John.2.22"
∷ word (ν ∷ ε ∷ κ ∷ ρ ∷ ῶ ∷ ν ∷ []) "John.2.22"
∷ word (ἐ ∷ μ ∷ ν ∷ ή ∷ σ ∷ θ ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.2.22"
∷ word (ο ∷ ἱ ∷ []) "John.2.22"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ α ∷ ὶ ∷ []) "John.2.22"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.2.22"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.2.22"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.2.22"
∷ word (ἔ ∷ ∙λ ∷ ε ∷ γ ∷ ε ∷ ν ∷ []) "John.2.22"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.2.22"
∷ word (ἐ ∷ π ∷ ί ∷ σ ∷ τ ∷ ε ∷ υ ∷ σ ∷ α ∷ ν ∷ []) "John.2.22"
∷ word (τ ∷ ῇ ∷ []) "John.2.22"
∷ word (γ ∷ ρ ∷ α ∷ φ ∷ ῇ ∷ []) "John.2.22"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.2.22"
∷ word (τ ∷ ῷ ∷ []) "John.2.22"
∷ word (∙λ ∷ ό ∷ γ ∷ ῳ ∷ []) "John.2.22"
∷ word (ὃ ∷ ν ∷ []) "John.2.22"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.2.22"
∷ word (ὁ ∷ []) "John.2.22"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.2.22"
∷ word (Ὡ ∷ ς ∷ []) "John.2.23"
∷ word (δ ∷ ὲ ∷ []) "John.2.23"
∷ word (ἦ ∷ ν ∷ []) "John.2.23"
∷ word (ἐ ∷ ν ∷ []) "John.2.23"
∷ word (τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.2.23"
∷ word (Ἱ ∷ ε ∷ ρ ∷ ο ∷ σ ∷ ο ∷ ∙λ ∷ ύ ∷ μ ∷ ο ∷ ι ∷ ς ∷ []) "John.2.23"
∷ word (ἐ ∷ ν ∷ []) "John.2.23"
∷ word (τ ∷ ῷ ∷ []) "John.2.23"
∷ word (π ∷ ά ∷ σ ∷ χ ∷ α ∷ []) "John.2.23"
∷ word (ἐ ∷ ν ∷ []) "John.2.23"
∷ word (τ ∷ ῇ ∷ []) "John.2.23"
∷ word (ἑ ∷ ο ∷ ρ ∷ τ ∷ ῇ ∷ []) "John.2.23"
∷ word (π ∷ ο ∷ ∙λ ∷ ∙λ ∷ ο ∷ ὶ ∷ []) "John.2.23"
∷ word (ἐ ∷ π ∷ ί ∷ σ ∷ τ ∷ ε ∷ υ ∷ σ ∷ α ∷ ν ∷ []) "John.2.23"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.2.23"
∷ word (τ ∷ ὸ ∷ []) "John.2.23"
∷ word (ὄ ∷ ν ∷ ο ∷ μ ∷ α ∷ []) "John.2.23"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.2.23"
∷ word (θ ∷ ε ∷ ω ∷ ρ ∷ ο ∷ ῦ ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.2.23"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.2.23"
∷ word (τ ∷ ὰ ∷ []) "John.2.23"
∷ word (σ ∷ η ∷ μ ∷ ε ∷ ῖ ∷ α ∷ []) "John.2.23"
∷ word (ἃ ∷ []) "John.2.23"
∷ word (ἐ ∷ π ∷ ο ∷ ί ∷ ε ∷ ι ∷ []) "John.2.23"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ς ∷ []) "John.2.24"
∷ word (δ ∷ ὲ ∷ []) "John.2.24"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.2.24"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.2.24"
∷ word (ἐ ∷ π ∷ ί ∷ σ ∷ τ ∷ ε ∷ υ ∷ ε ∷ ν ∷ []) "John.2.24"
∷ word (α ∷ ὑ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.2.24"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.2.24"
∷ word (δ ∷ ι ∷ ὰ ∷ []) "John.2.24"
∷ word (τ ∷ ὸ ∷ []) "John.2.24"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.2.24"
∷ word (γ ∷ ι ∷ ν ∷ ώ ∷ σ ∷ κ ∷ ε ∷ ι ∷ ν ∷ []) "John.2.24"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ α ∷ ς ∷ []) "John.2.24"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.2.25"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.2.25"
∷ word (ο ∷ ὐ ∷ []) "John.2.25"
∷ word (χ ∷ ρ ∷ ε ∷ ί ∷ α ∷ ν ∷ []) "John.2.25"
∷ word (ε ∷ ἶ ∷ χ ∷ ε ∷ ν ∷ []) "John.2.25"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.2.25"
∷ word (τ ∷ ι ∷ ς ∷ []) "John.2.25"
∷ word (μ ∷ α ∷ ρ ∷ τ ∷ υ ∷ ρ ∷ ή ∷ σ ∷ ῃ ∷ []) "John.2.25"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.2.25"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.2.25"
∷ word (ἀ ∷ ν ∷ θ ∷ ρ ∷ ώ ∷ π ∷ ο ∷ υ ∷ []) "John.2.25"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ς ∷ []) "John.2.25"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.2.25"
∷ word (ἐ ∷ γ ∷ ί ∷ ν ∷ ω ∷ σ ∷ κ ∷ ε ∷ ν ∷ []) "John.2.25"
∷ word (τ ∷ ί ∷ []) "John.2.25"
∷ word (ἦ ∷ ν ∷ []) "John.2.25"
∷ word (ἐ ∷ ν ∷ []) "John.2.25"
∷ word (τ ∷ ῷ ∷ []) "John.2.25"
∷ word (ἀ ∷ ν ∷ θ ∷ ρ ∷ ώ ∷ π ∷ ῳ ∷ []) "John.2.25"
∷ word (Ἦ ∷ ν ∷ []) "John.3.1"
∷ word (δ ∷ ὲ ∷ []) "John.3.1"
∷ word (ἄ ∷ ν ∷ θ ∷ ρ ∷ ω ∷ π ∷ ο ∷ ς ∷ []) "John.3.1"
∷ word (ἐ ∷ κ ∷ []) "John.3.1"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.3.1"
∷ word (Φ ∷ α ∷ ρ ∷ ι ∷ σ ∷ α ∷ ί ∷ ω ∷ ν ∷ []) "John.3.1"
∷ word (Ν ∷ ι ∷ κ ∷ ό ∷ δ ∷ η ∷ μ ∷ ο ∷ ς ∷ []) "John.3.1"
∷ word (ὄ ∷ ν ∷ ο ∷ μ ∷ α ∷ []) "John.3.1"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.3.1"
∷ word (ἄ ∷ ρ ∷ χ ∷ ω ∷ ν ∷ []) "John.3.1"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.3.1"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ί ∷ ω ∷ ν ∷ []) "John.3.1"
∷ word (ο ∷ ὗ ∷ τ ∷ ο ∷ ς ∷ []) "John.3.2"
∷ word (ἦ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.3.2"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.3.2"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.3.2"
∷ word (ν ∷ υ ∷ κ ∷ τ ∷ ὸ ∷ ς ∷ []) "John.3.2"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.3.2"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.3.2"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.3.2"
∷ word (Ῥ ∷ α ∷ β ∷ β ∷ ί ∷ []) "John.3.2"
∷ word (ο ∷ ἴ ∷ δ ∷ α ∷ μ ∷ ε ∷ ν ∷ []) "John.3.2"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.3.2"
∷ word (ἀ ∷ π ∷ ὸ ∷ []) "John.3.2"
∷ word (θ ∷ ε ∷ ο ∷ ῦ ∷ []) "John.3.2"
∷ word (ἐ ∷ ∙λ ∷ ή ∷ ∙λ ∷ υ ∷ θ ∷ α ∷ ς ∷ []) "John.3.2"
∷ word (δ ∷ ι ∷ δ ∷ ά ∷ σ ∷ κ ∷ α ∷ ∙λ ∷ ο ∷ ς ∷ []) "John.3.2"
∷ word (ο ∷ ὐ ∷ δ ∷ ε ∷ ὶ ∷ ς ∷ []) "John.3.2"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.3.2"
∷ word (δ ∷ ύ ∷ ν ∷ α ∷ τ ∷ α ∷ ι ∷ []) "John.3.2"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.3.2"
∷ word (τ ∷ ὰ ∷ []) "John.3.2"
∷ word (σ ∷ η ∷ μ ∷ ε ∷ ῖ ∷ α ∷ []) "John.3.2"
∷ word (π ∷ ο ∷ ι ∷ ε ∷ ῖ ∷ ν ∷ []) "John.3.2"
∷ word (ἃ ∷ []) "John.3.2"
∷ word (σ ∷ ὺ ∷ []) "John.3.2"
∷ word (π ∷ ο ∷ ι ∷ ε ∷ ῖ ∷ ς ∷ []) "John.3.2"
∷ word (ἐ ∷ ὰ ∷ ν ∷ []) "John.3.2"
∷ word (μ ∷ ὴ ∷ []) "John.3.2"
∷ word (ᾖ ∷ []) "John.3.2"
∷ word (ὁ ∷ []) "John.3.2"
∷ word (θ ∷ ε ∷ ὸ ∷ ς ∷ []) "John.3.2"
∷ word (μ ∷ ε ∷ τ ∷ []) "John.3.2"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.3.2"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.3.3"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.3.3"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.3.3"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.3.3"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.3.3"
∷ word (Ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.3.3"
∷ word (ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.3.3"
∷ word (∙λ ∷ έ ∷ γ ∷ ω ∷ []) "John.3.3"
∷ word (σ ∷ ο ∷ ι ∷ []) "John.3.3"
∷ word (ἐ ∷ ὰ ∷ ν ∷ []) "John.3.3"
∷ word (μ ∷ ή ∷ []) "John.3.3"
∷ word (τ ∷ ι ∷ ς ∷ []) "John.3.3"
∷ word (γ ∷ ε ∷ ν ∷ ν ∷ η ∷ θ ∷ ῇ ∷ []) "John.3.3"
∷ word (ἄ ∷ ν ∷ ω ∷ θ ∷ ε ∷ ν ∷ []) "John.3.3"
∷ word (ο ∷ ὐ ∷ []) "John.3.3"
∷ word (δ ∷ ύ ∷ ν ∷ α ∷ τ ∷ α ∷ ι ∷ []) "John.3.3"
∷ word (ἰ ∷ δ ∷ ε ∷ ῖ ∷ ν ∷ []) "John.3.3"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.3.3"
∷ word (β ∷ α ∷ σ ∷ ι ∷ ∙λ ∷ ε ∷ ί ∷ α ∷ ν ∷ []) "John.3.3"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.3.3"
∷ word (θ ∷ ε ∷ ο ∷ ῦ ∷ []) "John.3.3"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.3.4"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.3.4"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.3.4"
∷ word (ὁ ∷ []) "John.3.4"
∷ word (Ν ∷ ι ∷ κ ∷ ό ∷ δ ∷ η ∷ μ ∷ ο ∷ ς ∷ []) "John.3.4"
∷ word (Π ∷ ῶ ∷ ς ∷ []) "John.3.4"
∷ word (δ ∷ ύ ∷ ν ∷ α ∷ τ ∷ α ∷ ι ∷ []) "John.3.4"
∷ word (ἄ ∷ ν ∷ θ ∷ ρ ∷ ω ∷ π ∷ ο ∷ ς ∷ []) "John.3.4"
∷ word (γ ∷ ε ∷ ν ∷ ν ∷ η ∷ θ ∷ ῆ ∷ ν ∷ α ∷ ι ∷ []) "John.3.4"
∷ word (γ ∷ έ ∷ ρ ∷ ω ∷ ν ∷ []) "John.3.4"
∷ word (ὤ ∷ ν ∷ []) "John.3.4"
∷ word (μ ∷ ὴ ∷ []) "John.3.4"
∷ word (δ ∷ ύ ∷ ν ∷ α ∷ τ ∷ α ∷ ι ∷ []) "John.3.4"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.3.4"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.3.4"
∷ word (κ ∷ ο ∷ ι ∷ ∙λ ∷ ί ∷ α ∷ ν ∷ []) "John.3.4"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.3.4"
∷ word (μ ∷ η ∷ τ ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.3.4"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.3.4"
∷ word (δ ∷ ε ∷ ύ ∷ τ ∷ ε ∷ ρ ∷ ο ∷ ν ∷ []) "John.3.4"
∷ word (ε ∷ ἰ ∷ σ ∷ ε ∷ ∙λ ∷ θ ∷ ε ∷ ῖ ∷ ν ∷ []) "John.3.4"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.3.4"
∷ word (γ ∷ ε ∷ ν ∷ ν ∷ η ∷ θ ∷ ῆ ∷ ν ∷ α ∷ ι ∷ []) "John.3.4"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.3.5"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.3.5"
∷ word (Ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.3.5"
∷ word (ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.3.5"
∷ word (∙λ ∷ έ ∷ γ ∷ ω ∷ []) "John.3.5"
∷ word (σ ∷ ο ∷ ι ∷ []) "John.3.5"
∷ word (ἐ ∷ ὰ ∷ ν ∷ []) "John.3.5"
∷ word (μ ∷ ή ∷ []) "John.3.5"
∷ word (τ ∷ ι ∷ ς ∷ []) "John.3.5"
∷ word (γ ∷ ε ∷ ν ∷ ν ∷ η ∷ θ ∷ ῇ ∷ []) "John.3.5"
∷ word (ἐ ∷ ξ ∷ []) "John.3.5"
∷ word (ὕ ∷ δ ∷ α ∷ τ ∷ ο ∷ ς ∷ []) "John.3.5"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.3.5"
∷ word (π ∷ ν ∷ ε ∷ ύ ∷ μ ∷ α ∷ τ ∷ ο ∷ ς ∷ []) "John.3.5"
∷ word (ο ∷ ὐ ∷ []) "John.3.5"
∷ word (δ ∷ ύ ∷ ν ∷ α ∷ τ ∷ α ∷ ι ∷ []) "John.3.5"
∷ word (ε ∷ ἰ ∷ σ ∷ ε ∷ ∙λ ∷ θ ∷ ε ∷ ῖ ∷ ν ∷ []) "John.3.5"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.3.5"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.3.5"
∷ word (β ∷ α ∷ σ ∷ ι ∷ ∙λ ∷ ε ∷ ί ∷ α ∷ ν ∷ []) "John.3.5"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.3.5"
∷ word (θ ∷ ε ∷ ο ∷ ῦ ∷ []) "John.3.5"
∷ word (τ ∷ ὸ ∷ []) "John.3.6"
∷ word (γ ∷ ε ∷ γ ∷ ε ∷ ν ∷ ν ∷ η ∷ μ ∷ έ ∷ ν ∷ ο ∷ ν ∷ []) "John.3.6"
∷ word (ἐ ∷ κ ∷ []) "John.3.6"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.3.6"
∷ word (σ ∷ α ∷ ρ ∷ κ ∷ ὸ ∷ ς ∷ []) "John.3.6"
∷ word (σ ∷ ά ∷ ρ ∷ ξ ∷ []) "John.3.6"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.3.6"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.3.6"
∷ word (τ ∷ ὸ ∷ []) "John.3.6"
∷ word (γ ∷ ε ∷ γ ∷ ε ∷ ν ∷ ν ∷ η ∷ μ ∷ έ ∷ ν ∷ ο ∷ ν ∷ []) "John.3.6"
∷ word (ἐ ∷ κ ∷ []) "John.3.6"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.3.6"
∷ word (π ∷ ν ∷ ε ∷ ύ ∷ μ ∷ α ∷ τ ∷ ο ∷ ς ∷ []) "John.3.6"
∷ word (π ∷ ν ∷ ε ∷ ῦ ∷ μ ∷ ά ∷ []) "John.3.6"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.3.6"
∷ word (μ ∷ ὴ ∷ []) "John.3.7"
∷ word (θ ∷ α ∷ υ ∷ μ ∷ ά ∷ σ ∷ ῃ ∷ ς ∷ []) "John.3.7"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.3.7"
∷ word (ε ∷ ἶ ∷ π ∷ ό ∷ ν ∷ []) "John.3.7"
∷ word (σ ∷ ο ∷ ι ∷ []) "John.3.7"
∷ word (Δ ∷ ε ∷ ῖ ∷ []) "John.3.7"
∷ word (ὑ ∷ μ ∷ ᾶ ∷ ς ∷ []) "John.3.7"
∷ word (γ ∷ ε ∷ ν ∷ ν ∷ η ∷ θ ∷ ῆ ∷ ν ∷ α ∷ ι ∷ []) "John.3.7"
∷ word (ἄ ∷ ν ∷ ω ∷ θ ∷ ε ∷ ν ∷ []) "John.3.7"
∷ word (τ ∷ ὸ ∷ []) "John.3.8"
∷ word (π ∷ ν ∷ ε ∷ ῦ ∷ μ ∷ α ∷ []) "John.3.8"
∷ word (ὅ ∷ π ∷ ο ∷ υ ∷ []) "John.3.8"
∷ word (θ ∷ έ ∷ ∙λ ∷ ε ∷ ι ∷ []) "John.3.8"
∷ word (π ∷ ν ∷ ε ∷ ῖ ∷ []) "John.3.8"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.3.8"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.3.8"
∷ word (φ ∷ ω ∷ ν ∷ ὴ ∷ ν ∷ []) "John.3.8"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.3.8"
∷ word (ἀ ∷ κ ∷ ο ∷ ύ ∷ ε ∷ ι ∷ ς ∷ []) "John.3.8"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ []) "John.3.8"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.3.8"
∷ word (ο ∷ ἶ ∷ δ ∷ α ∷ ς ∷ []) "John.3.8"
∷ word (π ∷ ό ∷ θ ∷ ε ∷ ν ∷ []) "John.3.8"
∷ word (ἔ ∷ ρ ∷ χ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.3.8"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.3.8"
∷ word (π ∷ ο ∷ ῦ ∷ []) "John.3.8"
∷ word (ὑ ∷ π ∷ ά ∷ γ ∷ ε ∷ ι ∷ []) "John.3.8"
∷ word (ο ∷ ὕ ∷ τ ∷ ω ∷ ς ∷ []) "John.3.8"
∷ word (ἐ ∷ σ ∷ τ ∷ ὶ ∷ ν ∷ []) "John.3.8"
∷ word (π ∷ ᾶ ∷ ς ∷ []) "John.3.8"
∷ word (ὁ ∷ []) "John.3.8"
∷ word (γ ∷ ε ∷ γ ∷ ε ∷ ν ∷ ν ∷ η ∷ μ ∷ έ ∷ ν ∷ ο ∷ ς ∷ []) "John.3.8"
∷ word (ἐ ∷ κ ∷ []) "John.3.8"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.3.8"
∷ word (π ∷ ν ∷ ε ∷ ύ ∷ μ ∷ α ∷ τ ∷ ο ∷ ς ∷ []) "John.3.8"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.3.9"
∷ word (Ν ∷ ι ∷ κ ∷ ό ∷ δ ∷ η ∷ μ ∷ ο ∷ ς ∷ []) "John.3.9"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.3.9"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.3.9"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.3.9"
∷ word (Π ∷ ῶ ∷ ς ∷ []) "John.3.9"
∷ word (δ ∷ ύ ∷ ν ∷ α ∷ τ ∷ α ∷ ι ∷ []) "John.3.9"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.3.9"
∷ word (γ ∷ ε ∷ ν ∷ έ ∷ σ ∷ θ ∷ α ∷ ι ∷ []) "John.3.9"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.3.10"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.3.10"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.3.10"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.3.10"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.3.10"
∷ word (Σ ∷ ὺ ∷ []) "John.3.10"
∷ word (ε ∷ ἶ ∷ []) "John.3.10"
∷ word (ὁ ∷ []) "John.3.10"
∷ word (δ ∷ ι ∷ δ ∷ ά ∷ σ ∷ κ ∷ α ∷ ∙λ ∷ ο ∷ ς ∷ []) "John.3.10"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.3.10"
∷ word (Ἰ ∷ σ ∷ ρ ∷ α ∷ ὴ ∷ ∙λ ∷ []) "John.3.10"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.3.10"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.3.10"
∷ word (ο ∷ ὐ ∷ []) "John.3.10"
∷ word (γ ∷ ι ∷ ν ∷ ώ ∷ σ ∷ κ ∷ ε ∷ ι ∷ ς ∷ []) "John.3.10"
∷ word (ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.3.11"
∷ word (ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.3.11"
∷ word (∙λ ∷ έ ∷ γ ∷ ω ∷ []) "John.3.11"
∷ word (σ ∷ ο ∷ ι ∷ []) "John.3.11"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.3.11"
∷ word (ὃ ∷ []) "John.3.11"
∷ word (ο ∷ ἴ ∷ δ ∷ α ∷ μ ∷ ε ∷ ν ∷ []) "John.3.11"
∷ word (∙λ ∷ α ∷ ∙λ ∷ ο ∷ ῦ ∷ μ ∷ ε ∷ ν ∷ []) "John.3.11"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.3.11"
∷ word (ὃ ∷ []) "John.3.11"
∷ word (ἑ ∷ ω ∷ ρ ∷ ά ∷ κ ∷ α ∷ μ ∷ ε ∷ ν ∷ []) "John.3.11"
∷ word (μ ∷ α ∷ ρ ∷ τ ∷ υ ∷ ρ ∷ ο ∷ ῦ ∷ μ ∷ ε ∷ ν ∷ []) "John.3.11"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.3.11"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.3.11"
∷ word (μ ∷ α ∷ ρ ∷ τ ∷ υ ∷ ρ ∷ ί ∷ α ∷ ν ∷ []) "John.3.11"
∷ word (ἡ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.3.11"
∷ word (ο ∷ ὐ ∷ []) "John.3.11"
∷ word (∙λ ∷ α ∷ μ ∷ β ∷ ά ∷ ν ∷ ε ∷ τ ∷ ε ∷ []) "John.3.11"
∷ word (ε ∷ ἰ ∷ []) "John.3.12"
∷ word (τ ∷ ὰ ∷ []) "John.3.12"
∷ word (ἐ ∷ π ∷ ί ∷ γ ∷ ε ∷ ι ∷ α ∷ []) "John.3.12"
∷ word (ε ∷ ἶ ∷ π ∷ ο ∷ ν ∷ []) "John.3.12"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.3.12"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.3.12"
∷ word (ο ∷ ὐ ∷ []) "John.3.12"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ ε ∷ τ ∷ ε ∷ []) "John.3.12"
∷ word (π ∷ ῶ ∷ ς ∷ []) "John.3.12"
∷ word (ἐ ∷ ὰ ∷ ν ∷ []) "John.3.12"
∷ word (ε ∷ ἴ ∷ π ∷ ω ∷ []) "John.3.12"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.3.12"
∷ word (τ ∷ ὰ ∷ []) "John.3.12"
∷ word (ἐ ∷ π ∷ ο ∷ υ ∷ ρ ∷ ά ∷ ν ∷ ι ∷ α ∷ []) "John.3.12"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ σ ∷ ε ∷ τ ∷ ε ∷ []) "John.3.12"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.3.13"
∷ word (ο ∷ ὐ ∷ δ ∷ ε ∷ ὶ ∷ ς ∷ []) "John.3.13"
∷ word (ἀ ∷ ν ∷ α ∷ β ∷ έ ∷ β ∷ η ∷ κ ∷ ε ∷ ν ∷ []) "John.3.13"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.3.13"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.3.13"
∷ word (ο ∷ ὐ ∷ ρ ∷ α ∷ ν ∷ ὸ ∷ ν ∷ []) "John.3.13"
∷ word (ε ∷ ἰ ∷ []) "John.3.13"
∷ word (μ ∷ ὴ ∷ []) "John.3.13"
∷ word (ὁ ∷ []) "John.3.13"
∷ word (ἐ ∷ κ ∷ []) "John.3.13"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.3.13"
∷ word (ο ∷ ὐ ∷ ρ ∷ α ∷ ν ∷ ο ∷ ῦ ∷ []) "John.3.13"
∷ word (κ ∷ α ∷ τ ∷ α ∷ β ∷ ά ∷ ς ∷ []) "John.3.13"
∷ word (ὁ ∷ []) "John.3.13"
∷ word (υ ∷ ἱ ∷ ὸ ∷ ς ∷ []) "John.3.13"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.3.13"
∷ word (ἀ ∷ ν ∷ θ ∷ ρ ∷ ώ ∷ π ∷ ο ∷ υ ∷ []) "John.3.13"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.3.14"
∷ word (κ ∷ α ∷ θ ∷ ὼ ∷ ς ∷ []) "John.3.14"
∷ word (Μ ∷ ω ∷ ϋ ∷ σ ∷ ῆ ∷ ς ∷ []) "John.3.14"
∷ word (ὕ ∷ ψ ∷ ω ∷ σ ∷ ε ∷ ν ∷ []) "John.3.14"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.3.14"
∷ word (ὄ ∷ φ ∷ ι ∷ ν ∷ []) "John.3.14"
∷ word (ἐ ∷ ν ∷ []) "John.3.14"
∷ word (τ ∷ ῇ ∷ []) "John.3.14"
∷ word (ἐ ∷ ρ ∷ ή ∷ μ ∷ ῳ ∷ []) "John.3.14"
∷ word (ο ∷ ὕ ∷ τ ∷ ω ∷ ς ∷ []) "John.3.14"
∷ word (ὑ ∷ ψ ∷ ω ∷ θ ∷ ῆ ∷ ν ∷ α ∷ ι ∷ []) "John.3.14"
∷ word (δ ∷ ε ∷ ῖ ∷ []) "John.3.14"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.3.14"
∷ word (υ ∷ ἱ ∷ ὸ ∷ ν ∷ []) "John.3.14"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.3.14"
∷ word (ἀ ∷ ν ∷ θ ∷ ρ ∷ ώ ∷ π ∷ ο ∷ υ ∷ []) "John.3.14"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.3.15"
∷ word (π ∷ ᾶ ∷ ς ∷ []) "John.3.15"
∷ word (ὁ ∷ []) "John.3.15"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ ω ∷ ν ∷ []) "John.3.15"
∷ word (ἐ ∷ ν ∷ []) "John.3.15"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.3.15"
∷ word (ἔ ∷ χ ∷ ῃ ∷ []) "John.3.15"
∷ word (ζ ∷ ω ∷ ὴ ∷ ν ∷ []) "John.3.15"
∷ word (α ∷ ἰ ∷ ώ ∷ ν ∷ ι ∷ ο ∷ ν ∷ []) "John.3.15"
∷ word (Ο ∷ ὕ ∷ τ ∷ ω ∷ ς ∷ []) "John.3.16"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.3.16"
∷ word (ἠ ∷ γ ∷ ά ∷ π ∷ η ∷ σ ∷ ε ∷ ν ∷ []) "John.3.16"
∷ word (ὁ ∷ []) "John.3.16"
∷ word (θ ∷ ε ∷ ὸ ∷ ς ∷ []) "John.3.16"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.3.16"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ ν ∷ []) "John.3.16"
∷ word (ὥ ∷ σ ∷ τ ∷ ε ∷ []) "John.3.16"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.3.16"
∷ word (υ ∷ ἱ ∷ ὸ ∷ ν ∷ []) "John.3.16"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.3.16"
∷ word (μ ∷ ο ∷ ν ∷ ο ∷ γ ∷ ε ∷ ν ∷ ῆ ∷ []) "John.3.16"
∷ word (ἔ ∷ δ ∷ ω ∷ κ ∷ ε ∷ ν ∷ []) "John.3.16"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.3.16"
∷ word (π ∷ ᾶ ∷ ς ∷ []) "John.3.16"
∷ word (ὁ ∷ []) "John.3.16"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ ω ∷ ν ∷ []) "John.3.16"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.3.16"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.3.16"
∷ word (μ ∷ ὴ ∷ []) "John.3.16"
∷ word (ἀ ∷ π ∷ ό ∷ ∙λ ∷ η ∷ τ ∷ α ∷ ι ∷ []) "John.3.16"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.3.16"
∷ word (ἔ ∷ χ ∷ ῃ ∷ []) "John.3.16"
∷ word (ζ ∷ ω ∷ ὴ ∷ ν ∷ []) "John.3.16"
∷ word (α ∷ ἰ ∷ ώ ∷ ν ∷ ι ∷ ο ∷ ν ∷ []) "John.3.16"
∷ word (ο ∷ ὐ ∷ []) "John.3.17"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.3.17"
∷ word (ἀ ∷ π ∷ έ ∷ σ ∷ τ ∷ ε ∷ ι ∷ ∙λ ∷ ε ∷ ν ∷ []) "John.3.17"
∷ word (ὁ ∷ []) "John.3.17"
∷ word (θ ∷ ε ∷ ὸ ∷ ς ∷ []) "John.3.17"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.3.17"
∷ word (υ ∷ ἱ ∷ ὸ ∷ ν ∷ []) "John.3.17"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.3.17"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.3.17"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ ν ∷ []) "John.3.17"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.3.17"
∷ word (κ ∷ ρ ∷ ί ∷ ν ∷ ῃ ∷ []) "John.3.17"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.3.17"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ ν ∷ []) "John.3.17"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ []) "John.3.17"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.3.17"
∷ word (σ ∷ ω ∷ θ ∷ ῇ ∷ []) "John.3.17"
∷ word (ὁ ∷ []) "John.3.17"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ ς ∷ []) "John.3.17"
∷ word (δ ∷ ι ∷ []) "John.3.17"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.3.17"
∷ word (ὁ ∷ []) "John.3.18"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ ω ∷ ν ∷ []) "John.3.18"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.3.18"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.3.18"
∷ word (ο ∷ ὐ ∷ []) "John.3.18"
∷ word (κ ∷ ρ ∷ ί ∷ ν ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.3.18"
∷ word (ὁ ∷ []) "John.3.18"
∷ word (δ ∷ ὲ ∷ []) "John.3.18"
∷ word (μ ∷ ὴ ∷ []) "John.3.18"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ ω ∷ ν ∷ []) "John.3.18"
∷ word (ἤ ∷ δ ∷ η ∷ []) "John.3.18"
∷ word (κ ∷ έ ∷ κ ∷ ρ ∷ ι ∷ τ ∷ α ∷ ι ∷ []) "John.3.18"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.3.18"
∷ word (μ ∷ ὴ ∷ []) "John.3.18"
∷ word (π ∷ ε ∷ π ∷ ί ∷ σ ∷ τ ∷ ε ∷ υ ∷ κ ∷ ε ∷ ν ∷ []) "John.3.18"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.3.18"
∷ word (τ ∷ ὸ ∷ []) "John.3.18"
∷ word (ὄ ∷ ν ∷ ο ∷ μ ∷ α ∷ []) "John.3.18"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.3.18"
∷ word (μ ∷ ο ∷ ν ∷ ο ∷ γ ∷ ε ∷ ν ∷ ο ∷ ῦ ∷ ς ∷ []) "John.3.18"
∷ word (υ ∷ ἱ ∷ ο ∷ ῦ ∷ []) "John.3.18"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.3.18"
∷ word (θ ∷ ε ∷ ο ∷ ῦ ∷ []) "John.3.18"
∷ word (α ∷ ὕ ∷ τ ∷ η ∷ []) "John.3.19"
∷ word (δ ∷ έ ∷ []) "John.3.19"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.3.19"
∷ word (ἡ ∷ []) "John.3.19"
∷ word (κ ∷ ρ ∷ ί ∷ σ ∷ ι ∷ ς ∷ []) "John.3.19"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.3.19"
∷ word (τ ∷ ὸ ∷ []) "John.3.19"
∷ word (φ ∷ ῶ ∷ ς ∷ []) "John.3.19"
∷ word (ἐ ∷ ∙λ ∷ ή ∷ ∙λ ∷ υ ∷ θ ∷ ε ∷ ν ∷ []) "John.3.19"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.3.19"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.3.19"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ ν ∷ []) "John.3.19"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.3.19"
∷ word (ἠ ∷ γ ∷ ά ∷ π ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.3.19"
∷ word (ο ∷ ἱ ∷ []) "John.3.19"
∷ word (ἄ ∷ ν ∷ θ ∷ ρ ∷ ω ∷ π ∷ ο ∷ ι ∷ []) "John.3.19"
∷ word (μ ∷ ᾶ ∷ ∙λ ∷ ∙λ ∷ ο ∷ ν ∷ []) "John.3.19"
∷ word (τ ∷ ὸ ∷ []) "John.3.19"
∷ word (σ ∷ κ ∷ ό ∷ τ ∷ ο ∷ ς ∷ []) "John.3.19"
∷ word (ἢ ∷ []) "John.3.19"
∷ word (τ ∷ ὸ ∷ []) "John.3.19"
∷ word (φ ∷ ῶ ∷ ς ∷ []) "John.3.19"
∷ word (ἦ ∷ ν ∷ []) "John.3.19"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.3.19"
∷ word (α ∷ ὐ ∷ τ ∷ ῶ ∷ ν ∷ []) "John.3.19"
∷ word (π ∷ ο ∷ ν ∷ η ∷ ρ ∷ ὰ ∷ []) "John.3.19"
∷ word (τ ∷ ὰ ∷ []) "John.3.19"
∷ word (ἔ ∷ ρ ∷ γ ∷ α ∷ []) "John.3.19"
∷ word (π ∷ ᾶ ∷ ς ∷ []) "John.3.20"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.3.20"
∷ word (ὁ ∷ []) "John.3.20"
∷ word (φ ∷ α ∷ ῦ ∷ ∙λ ∷ α ∷ []) "John.3.20"
∷ word (π ∷ ρ ∷ ά ∷ σ ∷ σ ∷ ω ∷ ν ∷ []) "John.3.20"
∷ word (μ ∷ ι ∷ σ ∷ ε ∷ ῖ ∷ []) "John.3.20"
∷ word (τ ∷ ὸ ∷ []) "John.3.20"
∷ word (φ ∷ ῶ ∷ ς ∷ []) "John.3.20"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.3.20"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.3.20"
∷ word (ἔ ∷ ρ ∷ χ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.3.20"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.3.20"
∷ word (τ ∷ ὸ ∷ []) "John.3.20"
∷ word (φ ∷ ῶ ∷ ς ∷ []) "John.3.20"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.3.20"
∷ word (μ ∷ ὴ ∷ []) "John.3.20"
∷ word (ἐ ∷ ∙λ ∷ ε ∷ γ ∷ χ ∷ θ ∷ ῇ ∷ []) "John.3.20"
∷ word (τ ∷ ὰ ∷ []) "John.3.20"
∷ word (ἔ ∷ ρ ∷ γ ∷ α ∷ []) "John.3.20"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.3.20"
∷ word (ὁ ∷ []) "John.3.21"
∷ word (δ ∷ ὲ ∷ []) "John.3.21"
∷ word (π ∷ ο ∷ ι ∷ ῶ ∷ ν ∷ []) "John.3.21"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.3.21"
∷ word (ἀ ∷ ∙λ ∷ ή ∷ θ ∷ ε ∷ ι ∷ α ∷ ν ∷ []) "John.3.21"
∷ word (ἔ ∷ ρ ∷ χ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.3.21"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.3.21"
∷ word (τ ∷ ὸ ∷ []) "John.3.21"
∷ word (φ ∷ ῶ ∷ ς ∷ []) "John.3.21"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.3.21"
∷ word (φ ∷ α ∷ ν ∷ ε ∷ ρ ∷ ω ∷ θ ∷ ῇ ∷ []) "John.3.21"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.3.21"
∷ word (τ ∷ ὰ ∷ []) "John.3.21"
∷ word (ἔ ∷ ρ ∷ γ ∷ α ∷ []) "John.3.21"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.3.21"
∷ word (ἐ ∷ ν ∷ []) "John.3.21"
∷ word (θ ∷ ε ∷ ῷ ∷ []) "John.3.21"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.3.21"
∷ word (ε ∷ ἰ ∷ ρ ∷ γ ∷ α ∷ σ ∷ μ ∷ έ ∷ ν ∷ α ∷ []) "John.3.21"
∷ word (Μ ∷ ε ∷ τ ∷ ὰ ∷ []) "John.3.22"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.3.22"
∷ word (ἦ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.3.22"
∷ word (ὁ ∷ []) "John.3.22"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.3.22"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.3.22"
∷ word (ο ∷ ἱ ∷ []) "John.3.22"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ α ∷ ὶ ∷ []) "John.3.22"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.3.22"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.3.22"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.3.22"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ί ∷ α ∷ ν ∷ []) "John.3.22"
∷ word (γ ∷ ῆ ∷ ν ∷ []) "John.3.22"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.3.22"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ []) "John.3.22"
∷ word (δ ∷ ι ∷ έ ∷ τ ∷ ρ ∷ ι ∷ β ∷ ε ∷ ν ∷ []) "John.3.22"
∷ word (μ ∷ ε ∷ τ ∷ []) "John.3.22"
∷ word (α ∷ ὐ ∷ τ ∷ ῶ ∷ ν ∷ []) "John.3.22"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.3.22"
∷ word (ἐ ∷ β ∷ ά ∷ π ∷ τ ∷ ι ∷ ζ ∷ ε ∷ ν ∷ []) "John.3.22"
∷ word (ἦ ∷ ν ∷ []) "John.3.23"
∷ word (δ ∷ ὲ ∷ []) "John.3.23"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.3.23"
∷ word (ὁ ∷ []) "John.3.23"
∷ word (Ἰ ∷ ω ∷ ά ∷ ν ∷ ν ∷ η ∷ ς ∷ []) "John.3.23"
∷ word (β ∷ α ∷ π ∷ τ ∷ ί ∷ ζ ∷ ω ∷ ν ∷ []) "John.3.23"
∷ word (ἐ ∷ ν ∷ []) "John.3.23"
∷ word (Α ∷ ἰ ∷ ν ∷ ὼ ∷ ν ∷ []) "John.3.23"
∷ word (ἐ ∷ γ ∷ γ ∷ ὺ ∷ ς ∷ []) "John.3.23"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.3.23"
∷ word (Σ ∷ α ∷ ∙λ ∷ ε ∷ ί ∷ μ ∷ []) "John.3.23"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.3.23"
∷ word (ὕ ∷ δ ∷ α ∷ τ ∷ α ∷ []) "John.3.23"
∷ word (π ∷ ο ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.3.23"
∷ word (ἦ ∷ ν ∷ []) "John.3.23"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ []) "John.3.23"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.3.23"
∷ word (π ∷ α ∷ ρ ∷ ε ∷ γ ∷ ί ∷ ν ∷ ο ∷ ν ∷ τ ∷ ο ∷ []) "John.3.23"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.3.23"
∷ word (ἐ ∷ β ∷ α ∷ π ∷ τ ∷ ί ∷ ζ ∷ ο ∷ ν ∷ τ ∷ ο ∷ []) "John.3.23"
∷ word (ο ∷ ὔ ∷ π ∷ ω ∷ []) "John.3.24"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.3.24"
∷ word (ἦ ∷ ν ∷ []) "John.3.24"
∷ word (β ∷ ε ∷ β ∷ ∙λ ∷ η ∷ μ ∷ έ ∷ ν ∷ ο ∷ ς ∷ []) "John.3.24"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.3.24"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.3.24"
∷ word (φ ∷ υ ∷ ∙λ ∷ α ∷ κ ∷ ὴ ∷ ν ∷ []) "John.3.24"
∷ word (ὁ ∷ []) "John.3.24"
∷ word (Ἰ ∷ ω ∷ ά ∷ ν ∷ ν ∷ η ∷ ς ∷ []) "John.3.24"
∷ word (Ἐ ∷ γ ∷ έ ∷ ν ∷ ε ∷ τ ∷ ο ∷ []) "John.3.25"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.3.25"
∷ word (ζ ∷ ή ∷ τ ∷ η ∷ σ ∷ ι ∷ ς ∷ []) "John.3.25"
∷ word (ἐ ∷ κ ∷ []) "John.3.25"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.3.25"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ ῶ ∷ ν ∷ []) "John.3.25"
∷ word (Ἰ ∷ ω ∷ ά ∷ ν ∷ ν ∷ ο ∷ υ ∷ []) "John.3.25"
∷ word (μ ∷ ε ∷ τ ∷ ὰ ∷ []) "John.3.25"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ί ∷ ο ∷ υ ∷ []) "John.3.25"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.3.25"
∷ word (κ ∷ α ∷ θ ∷ α ∷ ρ ∷ ι ∷ σ ∷ μ ∷ ο ∷ ῦ ∷ []) "John.3.25"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.3.26"
∷ word (ἦ ∷ ∙λ ∷ θ ∷ ο ∷ ν ∷ []) "John.3.26"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.3.26"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.3.26"
∷ word (Ἰ ∷ ω ∷ ά ∷ ν ∷ ν ∷ η ∷ ν ∷ []) "John.3.26"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.3.26"
∷ word (ε ∷ ἶ ∷ π ∷ α ∷ ν ∷ []) "John.3.26"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.3.26"
∷ word (Ῥ ∷ α ∷ β ∷ β ∷ ί ∷ []) "John.3.26"
∷ word (ὃ ∷ ς ∷ []) "John.3.26"
∷ word (ἦ ∷ ν ∷ []) "John.3.26"
∷ word (μ ∷ ε ∷ τ ∷ ὰ ∷ []) "John.3.26"
∷ word (σ ∷ ο ∷ ῦ ∷ []) "John.3.26"
∷ word (π ∷ έ ∷ ρ ∷ α ∷ ν ∷ []) "John.3.26"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.3.26"
∷ word (Ἰ ∷ ο ∷ ρ ∷ δ ∷ ά ∷ ν ∷ ο ∷ υ ∷ []) "John.3.26"
∷ word (ᾧ ∷ []) "John.3.26"
∷ word (σ ∷ ὺ ∷ []) "John.3.26"
∷ word (μ ∷ ε ∷ μ ∷ α ∷ ρ ∷ τ ∷ ύ ∷ ρ ∷ η ∷ κ ∷ α ∷ ς ∷ []) "John.3.26"
∷ word (ἴ ∷ δ ∷ ε ∷ []) "John.3.26"
∷ word (ο ∷ ὗ ∷ τ ∷ ο ∷ ς ∷ []) "John.3.26"
∷ word (β ∷ α ∷ π ∷ τ ∷ ί ∷ ζ ∷ ε ∷ ι ∷ []) "John.3.26"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.3.26"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.3.26"
∷ word (ἔ ∷ ρ ∷ χ ∷ ο ∷ ν ∷ τ ∷ α ∷ ι ∷ []) "John.3.26"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.3.26"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.3.26"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.3.27"
∷ word (Ἰ ∷ ω ∷ ά ∷ ν ∷ ν ∷ η ∷ ς ∷ []) "John.3.27"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.3.27"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.3.27"
∷ word (Ο ∷ ὐ ∷ []) "John.3.27"
∷ word (δ ∷ ύ ∷ ν ∷ α ∷ τ ∷ α ∷ ι ∷ []) "John.3.27"
∷ word (ἄ ∷ ν ∷ θ ∷ ρ ∷ ω ∷ π ∷ ο ∷ ς ∷ []) "John.3.27"
∷ word (∙λ ∷ α ∷ μ ∷ β ∷ ά ∷ ν ∷ ε ∷ ι ∷ ν ∷ []) "John.3.27"
∷ word (ο ∷ ὐ ∷ δ ∷ ὲ ∷ []) "John.3.27"
∷ word (ἓ ∷ ν ∷ []) "John.3.27"
∷ word (ἐ ∷ ὰ ∷ ν ∷ []) "John.3.27"
∷ word (μ ∷ ὴ ∷ []) "John.3.27"
∷ word (ᾖ ∷ []) "John.3.27"
∷ word (δ ∷ ε ∷ δ ∷ ο ∷ μ ∷ έ ∷ ν ∷ ο ∷ ν ∷ []) "John.3.27"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.3.27"
∷ word (ἐ ∷ κ ∷ []) "John.3.27"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.3.27"
∷ word (ο ∷ ὐ ∷ ρ ∷ α ∷ ν ∷ ο ∷ ῦ ∷ []) "John.3.27"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ὶ ∷ []) "John.3.28"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.3.28"
∷ word (μ ∷ ο ∷ ι ∷ []) "John.3.28"
∷ word (μ ∷ α ∷ ρ ∷ τ ∷ υ ∷ ρ ∷ ε ∷ ῖ ∷ τ ∷ ε ∷ []) "John.3.28"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.3.28"
∷ word (ε ∷ ἶ ∷ π ∷ ο ∷ ν ∷ []) "John.3.28"
∷ word (Ο ∷ ὐ ∷ κ ∷ []) "John.3.28"
∷ word (ε ∷ ἰ ∷ μ ∷ ὶ ∷ []) "John.3.28"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.3.28"
∷ word (ὁ ∷ []) "John.3.28"
∷ word (χ ∷ ρ ∷ ι ∷ σ ∷ τ ∷ ό ∷ ς ∷ []) "John.3.28"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ []) "John.3.28"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.3.28"
∷ word (Ἀ ∷ π ∷ ε ∷ σ ∷ τ ∷ α ∷ ∙λ ∷ μ ∷ έ ∷ ν ∷ ο ∷ ς ∷ []) "John.3.28"
∷ word (ε ∷ ἰ ∷ μ ∷ ὶ ∷ []) "John.3.28"
∷ word (ἔ ∷ μ ∷ π ∷ ρ ∷ ο ∷ σ ∷ θ ∷ ε ∷ ν ∷ []) "John.3.28"
∷ word (ἐ ∷ κ ∷ ε ∷ ί ∷ ν ∷ ο ∷ υ ∷ []) "John.3.28"
∷ word (ὁ ∷ []) "John.3.29"
∷ word (ἔ ∷ χ ∷ ω ∷ ν ∷ []) "John.3.29"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.3.29"
∷ word (ν ∷ ύ ∷ μ ∷ φ ∷ η ∷ ν ∷ []) "John.3.29"
∷ word (ν ∷ υ ∷ μ ∷ φ ∷ ί ∷ ο ∷ ς ∷ []) "John.3.29"
∷ word (ἐ ∷ σ ∷ τ ∷ ί ∷ ν ∷ []) "John.3.29"
∷ word (ὁ ∷ []) "John.3.29"
∷ word (δ ∷ ὲ ∷ []) "John.3.29"
∷ word (φ ∷ ί ∷ ∙λ ∷ ο ∷ ς ∷ []) "John.3.29"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.3.29"
∷ word (ν ∷ υ ∷ μ ∷ φ ∷ ί ∷ ο ∷ υ ∷ []) "John.3.29"
∷ word (ὁ ∷ []) "John.3.29"
∷ word (ἑ ∷ σ ∷ τ ∷ η ∷ κ ∷ ὼ ∷ ς ∷ []) "John.3.29"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.3.29"
∷ word (ἀ ∷ κ ∷ ο ∷ ύ ∷ ω ∷ ν ∷ []) "John.3.29"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.3.29"
∷ word (χ ∷ α ∷ ρ ∷ ᾷ ∷ []) "John.3.29"
∷ word (χ ∷ α ∷ ί ∷ ρ ∷ ε ∷ ι ∷ []) "John.3.29"
∷ word (δ ∷ ι ∷ ὰ ∷ []) "John.3.29"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.3.29"
∷ word (φ ∷ ω ∷ ν ∷ ὴ ∷ ν ∷ []) "John.3.29"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.3.29"
∷ word (ν ∷ υ ∷ μ ∷ φ ∷ ί ∷ ο ∷ υ ∷ []) "John.3.29"
∷ word (α ∷ ὕ ∷ τ ∷ η ∷ []) "John.3.29"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.3.29"
∷ word (ἡ ∷ []) "John.3.29"
∷ word (χ ∷ α ∷ ρ ∷ ὰ ∷ []) "John.3.29"
∷ word (ἡ ∷ []) "John.3.29"
∷ word (ἐ ∷ μ ∷ ὴ ∷ []) "John.3.29"
∷ word (π ∷ ε ∷ π ∷ ∙λ ∷ ή ∷ ρ ∷ ω ∷ τ ∷ α ∷ ι ∷ []) "John.3.29"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ο ∷ ν ∷ []) "John.3.30"
∷ word (δ ∷ ε ∷ ῖ ∷ []) "John.3.30"
∷ word (α ∷ ὐ ∷ ξ ∷ ά ∷ ν ∷ ε ∷ ι ∷ ν ∷ []) "John.3.30"
∷ word (ἐ ∷ μ ∷ ὲ ∷ []) "John.3.30"
∷ word (δ ∷ ὲ ∷ []) "John.3.30"
∷ word (ἐ ∷ ∙λ ∷ α ∷ τ ∷ τ ∷ ο ∷ ῦ ∷ σ ∷ θ ∷ α ∷ ι ∷ []) "John.3.30"
∷ word (Ὁ ∷ []) "John.3.31"
∷ word (ἄ ∷ ν ∷ ω ∷ θ ∷ ε ∷ ν ∷ []) "John.3.31"
∷ word (ἐ ∷ ρ ∷ χ ∷ ό ∷ μ ∷ ε ∷ ν ∷ ο ∷ ς ∷ []) "John.3.31"
∷ word (ἐ ∷ π ∷ ά ∷ ν ∷ ω ∷ []) "John.3.31"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ ω ∷ ν ∷ []) "John.3.31"
∷ word (ἐ ∷ σ ∷ τ ∷ ί ∷ ν ∷ []) "John.3.31"
∷ word (ὁ ∷ []) "John.3.31"
∷ word (ὢ ∷ ν ∷ []) "John.3.31"
∷ word (ἐ ∷ κ ∷ []) "John.3.31"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.3.31"
∷ word (γ ∷ ῆ ∷ ς ∷ []) "John.3.31"
∷ word (ἐ ∷ κ ∷ []) "John.3.31"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.3.31"
∷ word (γ ∷ ῆ ∷ ς ∷ []) "John.3.31"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.3.31"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.3.31"
∷ word (ἐ ∷ κ ∷ []) "John.3.31"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.3.31"
∷ word (γ ∷ ῆ ∷ ς ∷ []) "John.3.31"
∷ word (∙λ ∷ α ∷ ∙λ ∷ ε ∷ ῖ ∷ []) "John.3.31"
∷ word (ὁ ∷ []) "John.3.31"
∷ word (ἐ ∷ κ ∷ []) "John.3.31"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.3.31"
∷ word (ο ∷ ὐ ∷ ρ ∷ α ∷ ν ∷ ο ∷ ῦ ∷ []) "John.3.31"
∷ word (ἐ ∷ ρ ∷ χ ∷ ό ∷ μ ∷ ε ∷ ν ∷ ο ∷ ς ∷ []) "John.3.31"
∷ word (ἐ ∷ π ∷ ά ∷ ν ∷ ω ∷ []) "John.3.31"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ ω ∷ ν ∷ []) "John.3.31"
∷ word (ἐ ∷ σ ∷ τ ∷ ί ∷ ν ∷ []) "John.3.31"
∷ word (ὃ ∷ []) "John.3.32"
∷ word (ἑ ∷ ώ ∷ ρ ∷ α ∷ κ ∷ ε ∷ ν ∷ []) "John.3.32"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.3.32"
∷ word (ἤ ∷ κ ∷ ο ∷ υ ∷ σ ∷ ε ∷ ν ∷ []) "John.3.32"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.3.32"
∷ word (μ ∷ α ∷ ρ ∷ τ ∷ υ ∷ ρ ∷ ε ∷ ῖ ∷ []) "John.3.32"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.3.32"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.3.32"
∷ word (μ ∷ α ∷ ρ ∷ τ ∷ υ ∷ ρ ∷ ί ∷ α ∷ ν ∷ []) "John.3.32"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.3.32"
∷ word (ο ∷ ὐ ∷ δ ∷ ε ∷ ὶ ∷ ς ∷ []) "John.3.32"
∷ word (∙λ ∷ α ∷ μ ∷ β ∷ ά ∷ ν ∷ ε ∷ ι ∷ []) "John.3.32"
∷ word (ὁ ∷ []) "John.3.33"
∷ word (∙λ ∷ α ∷ β ∷ ὼ ∷ ν ∷ []) "John.3.33"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.3.33"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.3.33"
∷ word (μ ∷ α ∷ ρ ∷ τ ∷ υ ∷ ρ ∷ ί ∷ α ∷ ν ∷ []) "John.3.33"
∷ word (ἐ ∷ σ ∷ φ ∷ ρ ∷ ά ∷ γ ∷ ι ∷ σ ∷ ε ∷ ν ∷ []) "John.3.33"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.3.33"
∷ word (ὁ ∷ []) "John.3.33"
∷ word (θ ∷ ε ∷ ὸ ∷ ς ∷ []) "John.3.33"
∷ word (ἀ ∷ ∙λ ∷ η ∷ θ ∷ ή ∷ ς ∷ []) "John.3.33"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.3.33"
∷ word (ὃ ∷ ν ∷ []) "John.3.34"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.3.34"
∷ word (ἀ ∷ π ∷ έ ∷ σ ∷ τ ∷ ε ∷ ι ∷ ∙λ ∷ ε ∷ ν ∷ []) "John.3.34"
∷ word (ὁ ∷ []) "John.3.34"
∷ word (θ ∷ ε ∷ ὸ ∷ ς ∷ []) "John.3.34"
∷ word (τ ∷ ὰ ∷ []) "John.3.34"
∷ word (ῥ ∷ ή ∷ μ ∷ α ∷ τ ∷ α ∷ []) "John.3.34"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.3.34"
∷ word (θ ∷ ε ∷ ο ∷ ῦ ∷ []) "John.3.34"
∷ word (∙λ ∷ α ∷ ∙λ ∷ ε ∷ ῖ ∷ []) "John.3.34"
∷ word (ο ∷ ὐ ∷ []) "John.3.34"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.3.34"
∷ word (ἐ ∷ κ ∷ []) "John.3.34"
∷ word (μ ∷ έ ∷ τ ∷ ρ ∷ ο ∷ υ ∷ []) "John.3.34"
∷ word (δ ∷ ί ∷ δ ∷ ω ∷ σ ∷ ι ∷ ν ∷ []) "John.3.34"
∷ word (τ ∷ ὸ ∷ []) "John.3.34"
∷ word (π ∷ ν ∷ ε ∷ ῦ ∷ μ ∷ α ∷ []) "John.3.34"
∷ word (ὁ ∷ []) "John.3.35"
∷ word (π ∷ α ∷ τ ∷ ὴ ∷ ρ ∷ []) "John.3.35"
∷ word (ἀ ∷ γ ∷ α ∷ π ∷ ᾷ ∷ []) "John.3.35"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.3.35"
∷ word (υ ∷ ἱ ∷ ό ∷ ν ∷ []) "John.3.35"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.3.35"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ α ∷ []) "John.3.35"
∷ word (δ ∷ έ ∷ δ ∷ ω ∷ κ ∷ ε ∷ ν ∷ []) "John.3.35"
∷ word (ἐ ∷ ν ∷ []) "John.3.35"
∷ word (τ ∷ ῇ ∷ []) "John.3.35"
∷ word (χ ∷ ε ∷ ι ∷ ρ ∷ ὶ ∷ []) "John.3.35"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.3.35"
∷ word (ὁ ∷ []) "John.3.36"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ ω ∷ ν ∷ []) "John.3.36"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.3.36"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.3.36"
∷ word (υ ∷ ἱ ∷ ὸ ∷ ν ∷ []) "John.3.36"
∷ word (ἔ ∷ χ ∷ ε ∷ ι ∷ []) "John.3.36"
∷ word (ζ ∷ ω ∷ ὴ ∷ ν ∷ []) "John.3.36"
∷ word (α ∷ ἰ ∷ ώ ∷ ν ∷ ι ∷ ο ∷ ν ∷ []) "John.3.36"
∷ word (ὁ ∷ []) "John.3.36"
∷ word (δ ∷ ὲ ∷ []) "John.3.36"
∷ word (ἀ ∷ π ∷ ε ∷ ι ∷ θ ∷ ῶ ∷ ν ∷ []) "John.3.36"
∷ word (τ ∷ ῷ ∷ []) "John.3.36"
∷ word (υ ∷ ἱ ∷ ῷ ∷ []) "John.3.36"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.3.36"
∷ word (ὄ ∷ ψ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.3.36"
∷ word (ζ ∷ ω ∷ ή ∷ ν ∷ []) "John.3.36"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ []) "John.3.36"
∷ word (ἡ ∷ []) "John.3.36"
∷ word (ὀ ∷ ρ ∷ γ ∷ ὴ ∷ []) "John.3.36"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.3.36"
∷ word (θ ∷ ε ∷ ο ∷ ῦ ∷ []) "John.3.36"
∷ word (μ ∷ έ ∷ ν ∷ ε ∷ ι ∷ []) "John.3.36"
∷ word (ἐ ∷ π ∷ []) "John.3.36"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.3.36"
∷ word (Ὡ ∷ ς ∷ []) "John.4.1"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.4.1"
∷ word (ἔ ∷ γ ∷ ν ∷ ω ∷ []) "John.4.1"
∷ word (ὁ ∷ []) "John.4.1"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.4.1"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.4.1"
∷ word (ἤ ∷ κ ∷ ο ∷ υ ∷ σ ∷ α ∷ ν ∷ []) "John.4.1"
∷ word (ο ∷ ἱ ∷ []) "John.4.1"
∷ word (Φ ∷ α ∷ ρ ∷ ι ∷ σ ∷ α ∷ ῖ ∷ ο ∷ ι ∷ []) "John.4.1"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.4.1"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.4.1"
∷ word (π ∷ ∙λ ∷ ε ∷ ί ∷ ο ∷ ν ∷ α ∷ ς ∷ []) "John.4.1"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ ὰ ∷ ς ∷ []) "John.4.1"
∷ word (π ∷ ο ∷ ι ∷ ε ∷ ῖ ∷ []) "John.4.1"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.4.1"
∷ word (β ∷ α ∷ π ∷ τ ∷ ί ∷ ζ ∷ ε ∷ ι ∷ []) "John.4.1"
∷ word (ἢ ∷ []) "John.4.1"
∷ word (Ἰ ∷ ω ∷ ά ∷ ν ∷ ν ∷ η ∷ ς ∷ []) "John.4.1"
∷ word (κ ∷ α ∷ ί ∷ τ ∷ ο ∷ ι ∷ γ ∷ ε ∷ []) "John.4.2"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.4.2"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ς ∷ []) "John.4.2"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.4.2"
∷ word (ἐ ∷ β ∷ ά ∷ π ∷ τ ∷ ι ∷ ζ ∷ ε ∷ ν ∷ []) "John.4.2"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ []) "John.4.2"
∷ word (ο ∷ ἱ ∷ []) "John.4.2"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ α ∷ ὶ ∷ []) "John.4.2"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.4.2"
∷ word (ἀ ∷ φ ∷ ῆ ∷ κ ∷ ε ∷ ν ∷ []) "John.4.3"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.4.3"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ί ∷ α ∷ ν ∷ []) "John.4.3"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.4.3"
∷ word (ἀ ∷ π ∷ ῆ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.4.3"
∷ word (π ∷ ά ∷ ∙λ ∷ ι ∷ ν ∷ []) "John.4.3"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.4.3"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.4.3"
∷ word (Γ ∷ α ∷ ∙λ ∷ ι ∷ ∙λ ∷ α ∷ ί ∷ α ∷ ν ∷ []) "John.4.3"
∷ word (ἔ ∷ δ ∷ ε ∷ ι ∷ []) "John.4.4"
∷ word (δ ∷ ὲ ∷ []) "John.4.4"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.4.4"
∷ word (δ ∷ ι ∷ έ ∷ ρ ∷ χ ∷ ε ∷ σ ∷ θ ∷ α ∷ ι ∷ []) "John.4.4"
∷ word (δ ∷ ι ∷ ὰ ∷ []) "John.4.4"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.4.4"
∷ word (Σ ∷ α ∷ μ ∷ α ∷ ρ ∷ ε ∷ ί ∷ α ∷ ς ∷ []) "John.4.4"
∷ word (ἔ ∷ ρ ∷ χ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.4.5"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.4.5"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.4.5"
∷ word (π ∷ ό ∷ ∙λ ∷ ι ∷ ν ∷ []) "John.4.5"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.4.5"
∷ word (Σ ∷ α ∷ μ ∷ α ∷ ρ ∷ ε ∷ ί ∷ α ∷ ς ∷ []) "John.4.5"
∷ word (∙λ ∷ ε ∷ γ ∷ ο ∷ μ ∷ έ ∷ ν ∷ η ∷ ν ∷ []) "John.4.5"
∷ word (Σ ∷ υ ∷ χ ∷ ὰ ∷ ρ ∷ []) "John.4.5"
∷ word (π ∷ ∙λ ∷ η ∷ σ ∷ ί ∷ ο ∷ ν ∷ []) "John.4.5"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.4.5"
∷ word (χ ∷ ω ∷ ρ ∷ ί ∷ ο ∷ υ ∷ []) "John.4.5"
∷ word (ὃ ∷ []) "John.4.5"
∷ word (ἔ ∷ δ ∷ ω ∷ κ ∷ ε ∷ ν ∷ []) "John.4.5"
∷ word (Ἰ ∷ α ∷ κ ∷ ὼ ∷ β ∷ []) "John.4.5"
∷ word (τ ∷ ῷ ∷ []) "John.4.5"
∷ word (Ἰ ∷ ω ∷ σ ∷ ὴ ∷ φ ∷ []) "John.4.5"
∷ word (τ ∷ ῷ ∷ []) "John.4.5"
∷ word (υ ∷ ἱ ∷ ῷ ∷ []) "John.4.5"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.4.5"
∷ word (ἦ ∷ ν ∷ []) "John.4.6"
∷ word (δ ∷ ὲ ∷ []) "John.4.6"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ []) "John.4.6"
∷ word (π ∷ η ∷ γ ∷ ὴ ∷ []) "John.4.6"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.4.6"
∷ word (Ἰ ∷ α ∷ κ ∷ ώ ∷ β ∷ []) "John.4.6"
∷ word (ὁ ∷ []) "John.4.6"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.4.6"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.4.6"
∷ word (κ ∷ ε ∷ κ ∷ ο ∷ π ∷ ι ∷ α ∷ κ ∷ ὼ ∷ ς ∷ []) "John.4.6"
∷ word (ἐ ∷ κ ∷ []) "John.4.6"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.4.6"
∷ word (ὁ ∷ δ ∷ ο ∷ ι ∷ π ∷ ο ∷ ρ ∷ ί ∷ α ∷ ς ∷ []) "John.4.6"
∷ word (ἐ ∷ κ ∷ α ∷ θ ∷ έ ∷ ζ ∷ ε ∷ τ ∷ ο ∷ []) "John.4.6"
∷ word (ο ∷ ὕ ∷ τ ∷ ω ∷ ς ∷ []) "John.4.6"
∷ word (ἐ ∷ π ∷ ὶ ∷ []) "John.4.6"
∷ word (τ ∷ ῇ ∷ []) "John.4.6"
∷ word (π ∷ η ∷ γ ∷ ῇ ∷ []) "John.4.6"
∷ word (ὥ ∷ ρ ∷ α ∷ []) "John.4.6"
∷ word (ἦ ∷ ν ∷ []) "John.4.6"
∷ word (ὡ ∷ ς ∷ []) "John.4.6"
∷ word (ἕ ∷ κ ∷ τ ∷ η ∷ []) "John.4.6"
∷ word (Ἔ ∷ ρ ∷ χ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.4.7"
∷ word (γ ∷ υ ∷ ν ∷ ὴ ∷ []) "John.4.7"
∷ word (ἐ ∷ κ ∷ []) "John.4.7"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.4.7"
∷ word (Σ ∷ α ∷ μ ∷ α ∷ ρ ∷ ε ∷ ί ∷ α ∷ ς ∷ []) "John.4.7"
∷ word (ἀ ∷ ν ∷ τ ∷ ∙λ ∷ ῆ ∷ σ ∷ α ∷ ι ∷ []) "John.4.7"
∷ word (ὕ ∷ δ ∷ ω ∷ ρ ∷ []) "John.4.7"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.4.7"
∷ word (α ∷ ὐ ∷ τ ∷ ῇ ∷ []) "John.4.7"
∷ word (ὁ ∷ []) "John.4.7"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.4.7"
∷ word (Δ ∷ ό ∷ ς ∷ []) "John.4.7"
∷ word (μ ∷ ο ∷ ι ∷ []) "John.4.7"
∷ word (π ∷ ε ∷ ῖ ∷ ν ∷ []) "John.4.7"
∷ word (ο ∷ ἱ ∷ []) "John.4.8"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.4.8"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ α ∷ ὶ ∷ []) "John.4.8"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.4.8"
∷ word (ἀ ∷ π ∷ ε ∷ ∙λ ∷ η ∷ ∙λ ∷ ύ ∷ θ ∷ ε ∷ ι ∷ σ ∷ α ∷ ν ∷ []) "John.4.8"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.4.8"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.4.8"
∷ word (π ∷ ό ∷ ∙λ ∷ ι ∷ ν ∷ []) "John.4.8"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.4.8"
∷ word (τ ∷ ρ ∷ ο ∷ φ ∷ ὰ ∷ ς ∷ []) "John.4.8"
∷ word (ἀ ∷ γ ∷ ο ∷ ρ ∷ ά ∷ σ ∷ ω ∷ σ ∷ ι ∷ ν ∷ []) "John.4.8"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.4.9"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.4.9"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.4.9"
∷ word (ἡ ∷ []) "John.4.9"
∷ word (γ ∷ υ ∷ ν ∷ ὴ ∷ []) "John.4.9"
∷ word (ἡ ∷ []) "John.4.9"
∷ word (Σ ∷ α ∷ μ ∷ α ∷ ρ ∷ ῖ ∷ τ ∷ ι ∷ ς ∷ []) "John.4.9"
∷ word (Π ∷ ῶ ∷ ς ∷ []) "John.4.9"
∷ word (σ ∷ ὺ ∷ []) "John.4.9"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ῖ ∷ ο ∷ ς ∷ []) "John.4.9"
∷ word (ὢ ∷ ν ∷ []) "John.4.9"
∷ word (π ∷ α ∷ ρ ∷ []) "John.4.9"
∷ word (ἐ ∷ μ ∷ ο ∷ ῦ ∷ []) "John.4.9"
∷ word (π ∷ ε ∷ ῖ ∷ ν ∷ []) "John.4.9"
∷ word (α ∷ ἰ ∷ τ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.4.9"
∷ word (γ ∷ υ ∷ ν ∷ α ∷ ι ∷ κ ∷ ὸ ∷ ς ∷ []) "John.4.9"
∷ word (Σ ∷ α ∷ μ ∷ α ∷ ρ ∷ ί ∷ τ ∷ ι ∷ δ ∷ ο ∷ ς ∷ []) "John.4.9"
∷ word (ο ∷ ὔ ∷ σ ∷ η ∷ ς ∷ []) "John.4.9"
∷ word (ο ∷ ὐ ∷ []) "John.4.9"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.4.9"
∷ word (σ ∷ υ ∷ γ ∷ χ ∷ ρ ∷ ῶ ∷ ν ∷ τ ∷ α ∷ ι ∷ []) "John.4.9"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ῖ ∷ ο ∷ ι ∷ []) "John.4.9"
∷ word (Σ ∷ α ∷ μ ∷ α ∷ ρ ∷ ί ∷ τ ∷ α ∷ ι ∷ ς ∷ []) "John.4.9"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.4.10"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.4.10"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.4.10"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.4.10"
∷ word (α ∷ ὐ ∷ τ ∷ ῇ ∷ []) "John.4.10"
∷ word (Ε ∷ ἰ ∷ []) "John.4.10"
∷ word (ᾔ ∷ δ ∷ ε ∷ ι ∷ ς ∷ []) "John.4.10"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.4.10"
∷ word (δ ∷ ω ∷ ρ ∷ ε ∷ ὰ ∷ ν ∷ []) "John.4.10"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.4.10"
∷ word (θ ∷ ε ∷ ο ∷ ῦ ∷ []) "John.4.10"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.4.10"
∷ word (τ ∷ ί ∷ ς ∷ []) "John.4.10"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.4.10"
∷ word (ὁ ∷ []) "John.4.10"
∷ word (∙λ ∷ έ ∷ γ ∷ ω ∷ ν ∷ []) "John.4.10"
∷ word (σ ∷ ο ∷ ι ∷ []) "John.4.10"
∷ word (Δ ∷ ό ∷ ς ∷ []) "John.4.10"
∷ word (μ ∷ ο ∷ ι ∷ []) "John.4.10"
∷ word (π ∷ ε ∷ ῖ ∷ ν ∷ []) "John.4.10"
∷ word (σ ∷ ὺ ∷ []) "John.4.10"
∷ word (ἂ ∷ ν ∷ []) "John.4.10"
∷ word (ᾔ ∷ τ ∷ η ∷ σ ∷ α ∷ ς ∷ []) "John.4.10"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.4.10"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.4.10"
∷ word (ἔ ∷ δ ∷ ω ∷ κ ∷ ε ∷ ν ∷ []) "John.4.10"
∷ word (ἄ ∷ ν ∷ []) "John.4.10"
∷ word (σ ∷ ο ∷ ι ∷ []) "John.4.10"
∷ word (ὕ ∷ δ ∷ ω ∷ ρ ∷ []) "John.4.10"
∷ word (ζ ∷ ῶ ∷ ν ∷ []) "John.4.10"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.4.11"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.4.11"
∷ word (ἡ ∷ []) "John.4.11"
∷ word (γ ∷ υ ∷ ν ∷ ή ∷ []) "John.4.11"
∷ word (Κ ∷ ύ ∷ ρ ∷ ι ∷ ε ∷ []) "John.4.11"
∷ word (ο ∷ ὔ ∷ τ ∷ ε ∷ []) "John.4.11"
∷ word (ἄ ∷ ν ∷ τ ∷ ∙λ ∷ η ∷ μ ∷ α ∷ []) "John.4.11"
∷ word (ἔ ∷ χ ∷ ε ∷ ι ∷ ς ∷ []) "John.4.11"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.4.11"
∷ word (τ ∷ ὸ ∷ []) "John.4.11"
∷ word (φ ∷ ρ ∷ έ ∷ α ∷ ρ ∷ []) "John.4.11"
∷ word (ἐ ∷ σ ∷ τ ∷ ὶ ∷ ν ∷ []) "John.4.11"
∷ word (β ∷ α ∷ θ ∷ ύ ∷ []) "John.4.11"
∷ word (π ∷ ό ∷ θ ∷ ε ∷ ν ∷ []) "John.4.11"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.4.11"
∷ word (ἔ ∷ χ ∷ ε ∷ ι ∷ ς ∷ []) "John.4.11"
∷ word (τ ∷ ὸ ∷ []) "John.4.11"
∷ word (ὕ ∷ δ ∷ ω ∷ ρ ∷ []) "John.4.11"
∷ word (τ ∷ ὸ ∷ []) "John.4.11"
∷ word (ζ ∷ ῶ ∷ ν ∷ []) "John.4.11"
∷ word (μ ∷ ὴ ∷ []) "John.4.12"
∷ word (σ ∷ ὺ ∷ []) "John.4.12"
∷ word (μ ∷ ε ∷ ί ∷ ζ ∷ ω ∷ ν ∷ []) "John.4.12"
∷ word (ε ∷ ἶ ∷ []) "John.4.12"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.4.12"
∷ word (π ∷ α ∷ τ ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.4.12"
∷ word (ἡ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.4.12"
∷ word (Ἰ ∷ α ∷ κ ∷ ώ ∷ β ∷ []) "John.4.12"
∷ word (ὃ ∷ ς ∷ []) "John.4.12"
∷ word (ἔ ∷ δ ∷ ω ∷ κ ∷ ε ∷ ν ∷ []) "John.4.12"
∷ word (ἡ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.4.12"
∷ word (τ ∷ ὸ ∷ []) "John.4.12"
∷ word (φ ∷ ρ ∷ έ ∷ α ∷ ρ ∷ []) "John.4.12"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.4.12"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ς ∷ []) "John.4.12"
∷ word (ἐ ∷ ξ ∷ []) "John.4.12"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.4.12"
∷ word (ἔ ∷ π ∷ ι ∷ ε ∷ ν ∷ []) "John.4.12"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.4.12"
∷ word (ο ∷ ἱ ∷ []) "John.4.12"
∷ word (υ ∷ ἱ ∷ ο ∷ ὶ ∷ []) "John.4.12"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.4.12"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.4.12"
∷ word (τ ∷ ὰ ∷ []) "John.4.12"
∷ word (θ ∷ ρ ∷ έ ∷ μ ∷ μ ∷ α ∷ τ ∷ α ∷ []) "John.4.12"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.4.12"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.4.13"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.4.13"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.4.13"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.4.13"
∷ word (α ∷ ὐ ∷ τ ∷ ῇ ∷ []) "John.4.13"
∷ word (Π ∷ ᾶ ∷ ς ∷ []) "John.4.13"
∷ word (ὁ ∷ []) "John.4.13"
∷ word (π ∷ ί ∷ ν ∷ ω ∷ ν ∷ []) "John.4.13"
∷ word (ἐ ∷ κ ∷ []) "John.4.13"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.4.13"
∷ word (ὕ ∷ δ ∷ α ∷ τ ∷ ο ∷ ς ∷ []) "John.4.13"
∷ word (τ ∷ ο ∷ ύ ∷ τ ∷ ο ∷ υ ∷ []) "John.4.13"
∷ word (δ ∷ ι ∷ ψ ∷ ή ∷ σ ∷ ε ∷ ι ∷ []) "John.4.13"
∷ word (π ∷ ά ∷ ∙λ ∷ ι ∷ ν ∷ []) "John.4.13"
∷ word (ὃ ∷ ς ∷ []) "John.4.14"
∷ word (δ ∷ []) "John.4.14"
∷ word (ἂ ∷ ν ∷ []) "John.4.14"
∷ word (π ∷ ί ∷ ῃ ∷ []) "John.4.14"
∷ word (ἐ ∷ κ ∷ []) "John.4.14"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.4.14"
∷ word (ὕ ∷ δ ∷ α ∷ τ ∷ ο ∷ ς ∷ []) "John.4.14"
∷ word (ο ∷ ὗ ∷ []) "John.4.14"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.4.14"
∷ word (δ ∷ ώ ∷ σ ∷ ω ∷ []) "John.4.14"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.4.14"
∷ word (ο ∷ ὐ ∷ []) "John.4.14"
∷ word (μ ∷ ὴ ∷ []) "John.4.14"
∷ word (δ ∷ ι ∷ ψ ∷ ή ∷ σ ∷ ε ∷ ι ∷ []) "John.4.14"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.4.14"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.4.14"
∷ word (α ∷ ἰ ∷ ῶ ∷ ν ∷ α ∷ []) "John.4.14"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.4.14"
∷ word (τ ∷ ὸ ∷ []) "John.4.14"
∷ word (ὕ ∷ δ ∷ ω ∷ ρ ∷ []) "John.4.14"
∷ word (ὃ ∷ []) "John.4.14"
∷ word (δ ∷ ώ ∷ σ ∷ ω ∷ []) "John.4.14"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.4.14"
∷ word (γ ∷ ε ∷ ν ∷ ή ∷ σ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.4.14"
∷ word (ἐ ∷ ν ∷ []) "John.4.14"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.4.14"
∷ word (π ∷ η ∷ γ ∷ ὴ ∷ []) "John.4.14"
∷ word (ὕ ∷ δ ∷ α ∷ τ ∷ ο ∷ ς ∷ []) "John.4.14"
∷ word (ἁ ∷ ∙λ ∷ ∙λ ∷ ο ∷ μ ∷ έ ∷ ν ∷ ο ∷ υ ∷ []) "John.4.14"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.4.14"
∷ word (ζ ∷ ω ∷ ὴ ∷ ν ∷ []) "John.4.14"
∷ word (α ∷ ἰ ∷ ώ ∷ ν ∷ ι ∷ ο ∷ ν ∷ []) "John.4.14"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.4.15"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.4.15"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.4.15"
∷ word (ἡ ∷ []) "John.4.15"
∷ word (γ ∷ υ ∷ ν ∷ ή ∷ []) "John.4.15"
∷ word (Κ ∷ ύ ∷ ρ ∷ ι ∷ ε ∷ []) "John.4.15"
∷ word (δ ∷ ό ∷ ς ∷ []) "John.4.15"
∷ word (μ ∷ ο ∷ ι ∷ []) "John.4.15"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.4.15"
∷ word (τ ∷ ὸ ∷ []) "John.4.15"
∷ word (ὕ ∷ δ ∷ ω ∷ ρ ∷ []) "John.4.15"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.4.15"
∷ word (μ ∷ ὴ ∷ []) "John.4.15"
∷ word (δ ∷ ι ∷ ψ ∷ ῶ ∷ []) "John.4.15"
∷ word (μ ∷ η ∷ δ ∷ ὲ ∷ []) "John.4.15"
∷ word (δ ∷ ι ∷ έ ∷ ρ ∷ χ ∷ ω ∷ μ ∷ α ∷ ι ∷ []) "John.4.15"
∷ word (ἐ ∷ ν ∷ θ ∷ ά ∷ δ ∷ ε ∷ []) "John.4.15"
∷ word (ἀ ∷ ν ∷ τ ∷ ∙λ ∷ ε ∷ ῖ ∷ ν ∷ []) "John.4.15"
∷ word (Λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.4.16"
∷ word (α ∷ ὐ ∷ τ ∷ ῇ ∷ []) "John.4.16"
∷ word (Ὕ ∷ π ∷ α ∷ γ ∷ ε ∷ []) "John.4.16"
∷ word (φ ∷ ώ ∷ ν ∷ η ∷ σ ∷ ο ∷ ν ∷ []) "John.4.16"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.4.16"
∷ word (ἄ ∷ ν ∷ δ ∷ ρ ∷ α ∷ []) "John.4.16"
∷ word (σ ∷ ο ∷ υ ∷ []) "John.4.16"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.4.16"
∷ word (ἐ ∷ ∙λ ∷ θ ∷ ὲ ∷ []) "John.4.16"
∷ word (ἐ ∷ ν ∷ θ ∷ ά ∷ δ ∷ ε ∷ []) "John.4.16"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.4.17"
∷ word (ἡ ∷ []) "John.4.17"
∷ word (γ ∷ υ ∷ ν ∷ ὴ ∷ []) "John.4.17"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.4.17"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.4.17"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.4.17"
∷ word (Ο ∷ ὐ ∷ κ ∷ []) "John.4.17"
∷ word (ἔ ∷ χ ∷ ω ∷ []) "John.4.17"
∷ word (ἄ ∷ ν ∷ δ ∷ ρ ∷ α ∷ []) "John.4.17"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.4.17"
∷ word (α ∷ ὐ ∷ τ ∷ ῇ ∷ []) "John.4.17"
∷ word (ὁ ∷ []) "John.4.17"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.4.17"
∷ word (Κ ∷ α ∷ ∙λ ∷ ῶ ∷ ς ∷ []) "John.4.17"
∷ word (ε ∷ ἶ ∷ π ∷ α ∷ ς ∷ []) "John.4.17"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.4.17"
∷ word (Ἄ ∷ ν ∷ δ ∷ ρ ∷ α ∷ []) "John.4.17"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.4.17"
∷ word (ἔ ∷ χ ∷ ω ∷ []) "John.4.17"
∷ word (π ∷ έ ∷ ν ∷ τ ∷ ε ∷ []) "John.4.18"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.4.18"
∷ word (ἄ ∷ ν ∷ δ ∷ ρ ∷ α ∷ ς ∷ []) "John.4.18"
∷ word (ἔ ∷ σ ∷ χ ∷ ε ∷ ς ∷ []) "John.4.18"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.4.18"
∷ word (ν ∷ ῦ ∷ ν ∷ []) "John.4.18"
∷ word (ὃ ∷ ν ∷ []) "John.4.18"
∷ word (ἔ ∷ χ ∷ ε ∷ ι ∷ ς ∷ []) "John.4.18"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.4.18"
∷ word (ἔ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.4.18"
∷ word (σ ∷ ο ∷ υ ∷ []) "John.4.18"
∷ word (ἀ ∷ ν ∷ ή ∷ ρ ∷ []) "John.4.18"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.4.18"
∷ word (ἀ ∷ ∙λ ∷ η ∷ θ ∷ ὲ ∷ ς ∷ []) "John.4.18"
∷ word (ε ∷ ἴ ∷ ρ ∷ η ∷ κ ∷ α ∷ ς ∷ []) "John.4.18"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.4.19"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.4.19"
∷ word (ἡ ∷ []) "John.4.19"
∷ word (γ ∷ υ ∷ ν ∷ ή ∷ []) "John.4.19"
∷ word (Κ ∷ ύ ∷ ρ ∷ ι ∷ ε ∷ []) "John.4.19"
∷ word (θ ∷ ε ∷ ω ∷ ρ ∷ ῶ ∷ []) "John.4.19"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.4.19"
∷ word (π ∷ ρ ∷ ο ∷ φ ∷ ή ∷ τ ∷ η ∷ ς ∷ []) "John.4.19"
∷ word (ε ∷ ἶ ∷ []) "John.4.19"
∷ word (σ ∷ ύ ∷ []) "John.4.19"
∷ word (ο ∷ ἱ ∷ []) "John.4.20"
∷ word (π ∷ α ∷ τ ∷ έ ∷ ρ ∷ ε ∷ ς ∷ []) "John.4.20"
∷ word (ἡ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.4.20"
∷ word (ἐ ∷ ν ∷ []) "John.4.20"
∷ word (τ ∷ ῷ ∷ []) "John.4.20"
∷ word (ὄ ∷ ρ ∷ ε ∷ ι ∷ []) "John.4.20"
∷ word (τ ∷ ο ∷ ύ ∷ τ ∷ ῳ ∷ []) "John.4.20"
∷ word (π ∷ ρ ∷ ο ∷ σ ∷ ε ∷ κ ∷ ύ ∷ ν ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.4.20"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.4.20"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.4.20"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ τ ∷ ε ∷ []) "John.4.20"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.4.20"
∷ word (ἐ ∷ ν ∷ []) "John.4.20"
∷ word (Ἱ ∷ ε ∷ ρ ∷ ο ∷ σ ∷ ο ∷ ∙λ ∷ ύ ∷ μ ∷ ο ∷ ι ∷ ς ∷ []) "John.4.20"
∷ word (ἐ ∷ σ ∷ τ ∷ ὶ ∷ ν ∷ []) "John.4.20"
∷ word (ὁ ∷ []) "John.4.20"
∷ word (τ ∷ ό ∷ π ∷ ο ∷ ς ∷ []) "John.4.20"
∷ word (ὅ ∷ π ∷ ο ∷ υ ∷ []) "John.4.20"
∷ word (π ∷ ρ ∷ ο ∷ σ ∷ κ ∷ υ ∷ ν ∷ ε ∷ ῖ ∷ ν ∷ []) "John.4.20"
∷ word (δ ∷ ε ∷ ῖ ∷ []) "John.4.20"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.4.21"
∷ word (α ∷ ὐ ∷ τ ∷ ῇ ∷ []) "John.4.21"
∷ word (ὁ ∷ []) "John.4.21"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.4.21"
∷ word (Π ∷ ί ∷ σ ∷ τ ∷ ε ∷ υ ∷ έ ∷ []) "John.4.21"
∷ word (μ ∷ ο ∷ ι ∷ []) "John.4.21"
∷ word (γ ∷ ύ ∷ ν ∷ α ∷ ι ∷ []) "John.4.21"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.4.21"
∷ word (ἔ ∷ ρ ∷ χ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.4.21"
∷ word (ὥ ∷ ρ ∷ α ∷ []) "John.4.21"
∷ word (ὅ ∷ τ ∷ ε ∷ []) "John.4.21"
∷ word (ο ∷ ὔ ∷ τ ∷ ε ∷ []) "John.4.21"
∷ word (ἐ ∷ ν ∷ []) "John.4.21"
∷ word (τ ∷ ῷ ∷ []) "John.4.21"
∷ word (ὄ ∷ ρ ∷ ε ∷ ι ∷ []) "John.4.21"
∷ word (τ ∷ ο ∷ ύ ∷ τ ∷ ῳ ∷ []) "John.4.21"
∷ word (ο ∷ ὔ ∷ τ ∷ ε ∷ []) "John.4.21"
∷ word (ἐ ∷ ν ∷ []) "John.4.21"
∷ word (Ἱ ∷ ε ∷ ρ ∷ ο ∷ σ ∷ ο ∷ ∙λ ∷ ύ ∷ μ ∷ ο ∷ ι ∷ ς ∷ []) "John.4.21"
∷ word (π ∷ ρ ∷ ο ∷ σ ∷ κ ∷ υ ∷ ν ∷ ή ∷ σ ∷ ε ∷ τ ∷ ε ∷ []) "John.4.21"
∷ word (τ ∷ ῷ ∷ []) "John.4.21"
∷ word (π ∷ α ∷ τ ∷ ρ ∷ ί ∷ []) "John.4.21"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.4.22"
∷ word (π ∷ ρ ∷ ο ∷ σ ∷ κ ∷ υ ∷ ν ∷ ε ∷ ῖ ∷ τ ∷ ε ∷ []) "John.4.22"
∷ word (ὃ ∷ []) "John.4.22"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.4.22"
∷ word (ο ∷ ἴ ∷ δ ∷ α ∷ τ ∷ ε ∷ []) "John.4.22"
∷ word (ἡ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.4.22"
∷ word (π ∷ ρ ∷ ο ∷ σ ∷ κ ∷ υ ∷ ν ∷ ο ∷ ῦ ∷ μ ∷ ε ∷ ν ∷ []) "John.4.22"
∷ word (ὃ ∷ []) "John.4.22"
∷ word (ο ∷ ἴ ∷ δ ∷ α ∷ μ ∷ ε ∷ ν ∷ []) "John.4.22"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.4.22"
∷ word (ἡ ∷ []) "John.4.22"
∷ word (σ ∷ ω ∷ τ ∷ η ∷ ρ ∷ ί ∷ α ∷ []) "John.4.22"
∷ word (ἐ ∷ κ ∷ []) "John.4.22"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.4.22"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ί ∷ ω ∷ ν ∷ []) "John.4.22"
∷ word (ἐ ∷ σ ∷ τ ∷ ί ∷ ν ∷ []) "John.4.22"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.4.23"
∷ word (ἔ ∷ ρ ∷ χ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.4.23"
∷ word (ὥ ∷ ρ ∷ α ∷ []) "John.4.23"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.4.23"
∷ word (ν ∷ ῦ ∷ ν ∷ []) "John.4.23"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.4.23"
∷ word (ὅ ∷ τ ∷ ε ∷ []) "John.4.23"
∷ word (ο ∷ ἱ ∷ []) "John.4.23"
∷ word (ἀ ∷ ∙λ ∷ η ∷ θ ∷ ι ∷ ν ∷ ο ∷ ὶ ∷ []) "John.4.23"
∷ word (π ∷ ρ ∷ ο ∷ σ ∷ κ ∷ υ ∷ ν ∷ η ∷ τ ∷ α ∷ ὶ ∷ []) "John.4.23"
∷ word (π ∷ ρ ∷ ο ∷ σ ∷ κ ∷ υ ∷ ν ∷ ή ∷ σ ∷ ο ∷ υ ∷ σ ∷ ι ∷ ν ∷ []) "John.4.23"
∷ word (τ ∷ ῷ ∷ []) "John.4.23"
∷ word (π ∷ α ∷ τ ∷ ρ ∷ ὶ ∷ []) "John.4.23"
∷ word (ἐ ∷ ν ∷ []) "John.4.23"
∷ word (π ∷ ν ∷ ε ∷ ύ ∷ μ ∷ α ∷ τ ∷ ι ∷ []) "John.4.23"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.4.23"
∷ word (ἀ ∷ ∙λ ∷ η ∷ θ ∷ ε ∷ ί ∷ ᾳ ∷ []) "John.4.23"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.4.23"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.4.23"
∷ word (ὁ ∷ []) "John.4.23"
∷ word (π ∷ α ∷ τ ∷ ὴ ∷ ρ ∷ []) "John.4.23"
∷ word (τ ∷ ο ∷ ι ∷ ο ∷ ύ ∷ τ ∷ ο ∷ υ ∷ ς ∷ []) "John.4.23"
∷ word (ζ ∷ η ∷ τ ∷ ε ∷ ῖ ∷ []) "John.4.23"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.4.23"
∷ word (π ∷ ρ ∷ ο ∷ σ ∷ κ ∷ υ ∷ ν ∷ ο ∷ ῦ ∷ ν ∷ τ ∷ α ∷ ς ∷ []) "John.4.23"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.4.23"
∷ word (π ∷ ν ∷ ε ∷ ῦ ∷ μ ∷ α ∷ []) "John.4.24"
∷ word (ὁ ∷ []) "John.4.24"
∷ word (θ ∷ ε ∷ ό ∷ ς ∷ []) "John.4.24"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.4.24"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.4.24"
∷ word (π ∷ ρ ∷ ο ∷ σ ∷ κ ∷ υ ∷ ν ∷ ο ∷ ῦ ∷ ν ∷ τ ∷ α ∷ ς ∷ []) "John.4.24"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.4.24"
∷ word (ἐ ∷ ν ∷ []) "John.4.24"
∷ word (π ∷ ν ∷ ε ∷ ύ ∷ μ ∷ α ∷ τ ∷ ι ∷ []) "John.4.24"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.4.24"
∷ word (ἀ ∷ ∙λ ∷ η ∷ θ ∷ ε ∷ ί ∷ ᾳ ∷ []) "John.4.24"
∷ word (δ ∷ ε ∷ ῖ ∷ []) "John.4.24"
∷ word (π ∷ ρ ∷ ο ∷ σ ∷ κ ∷ υ ∷ ν ∷ ε ∷ ῖ ∷ ν ∷ []) "John.4.24"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.4.25"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.4.25"
∷ word (ἡ ∷ []) "John.4.25"
∷ word (γ ∷ υ ∷ ν ∷ ή ∷ []) "John.4.25"
∷ word (Ο ∷ ἶ ∷ δ ∷ α ∷ []) "John.4.25"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.4.25"
∷ word (Μ ∷ ε ∷ σ ∷ σ ∷ ί ∷ α ∷ ς ∷ []) "John.4.25"
∷ word (ἔ ∷ ρ ∷ χ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.4.25"
∷ word (ὁ ∷ []) "John.4.25"
∷ word (∙λ ∷ ε ∷ γ ∷ ό ∷ μ ∷ ε ∷ ν ∷ ο ∷ ς ∷ []) "John.4.25"
∷ word (χ ∷ ρ ∷ ι ∷ σ ∷ τ ∷ ό ∷ ς ∷ []) "John.4.25"
∷ word (ὅ ∷ τ ∷ α ∷ ν ∷ []) "John.4.25"
∷ word (ἔ ∷ ∙λ ∷ θ ∷ ῃ ∷ []) "John.4.25"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ο ∷ ς ∷ []) "John.4.25"
∷ word (ἀ ∷ ν ∷ α ∷ γ ∷ γ ∷ ε ∷ ∙λ ∷ ε ∷ ῖ ∷ []) "John.4.25"
∷ word (ἡ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.4.25"
∷ word (ἅ ∷ π ∷ α ∷ ν ∷ τ ∷ α ∷ []) "John.4.25"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.4.26"
∷ word (α ∷ ὐ ∷ τ ∷ ῇ ∷ []) "John.4.26"
∷ word (ὁ ∷ []) "John.4.26"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.4.26"
∷ word (Ἐ ∷ γ ∷ ώ ∷ []) "John.4.26"
∷ word (ε ∷ ἰ ∷ μ ∷ ι ∷ []) "John.4.26"
∷ word (ὁ ∷ []) "John.4.26"
∷ word (∙λ ∷ α ∷ ∙λ ∷ ῶ ∷ ν ∷ []) "John.4.26"
∷ word (σ ∷ ο ∷ ι ∷ []) "John.4.26"
∷ word (Κ ∷ α ∷ ὶ ∷ []) "John.4.27"
∷ word (ἐ ∷ π ∷ ὶ ∷ []) "John.4.27"
∷ word (τ ∷ ο ∷ ύ ∷ τ ∷ ῳ ∷ []) "John.4.27"
∷ word (ἦ ∷ ∙λ ∷ θ ∷ α ∷ ν ∷ []) "John.4.27"
∷ word (ο ∷ ἱ ∷ []) "John.4.27"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ α ∷ ὶ ∷ []) "John.4.27"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.4.27"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.4.27"
∷ word (ἐ ∷ θ ∷ α ∷ ύ ∷ μ ∷ α ∷ ζ ∷ ο ∷ ν ∷ []) "John.4.27"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.4.27"
∷ word (μ ∷ ε ∷ τ ∷ ὰ ∷ []) "John.4.27"
∷ word (γ ∷ υ ∷ ν ∷ α ∷ ι ∷ κ ∷ ὸ ∷ ς ∷ []) "John.4.27"
∷ word (ἐ ∷ ∙λ ∷ ά ∷ ∙λ ∷ ε ∷ ι ∷ []) "John.4.27"
∷ word (ο ∷ ὐ ∷ δ ∷ ε ∷ ὶ ∷ ς ∷ []) "John.4.27"
∷ word (μ ∷ έ ∷ ν ∷ τ ∷ ο ∷ ι ∷ []) "John.4.27"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.4.27"
∷ word (Τ ∷ ί ∷ []) "John.4.27"
∷ word (ζ ∷ η ∷ τ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.4.27"
∷ word (ἢ ∷ []) "John.4.27"
∷ word (τ ∷ ί ∷ []) "John.4.27"
∷ word (∙λ ∷ α ∷ ∙λ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.4.27"
∷ word (μ ∷ ε ∷ τ ∷ []) "John.4.27"
∷ word (α ∷ ὐ ∷ τ ∷ ῆ ∷ ς ∷ []) "John.4.27"
∷ word (ἀ ∷ φ ∷ ῆ ∷ κ ∷ ε ∷ ν ∷ []) "John.4.28"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.4.28"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.4.28"
∷ word (ὑ ∷ δ ∷ ρ ∷ ί ∷ α ∷ ν ∷ []) "John.4.28"
∷ word (α ∷ ὐ ∷ τ ∷ ῆ ∷ ς ∷ []) "John.4.28"
∷ word (ἡ ∷ []) "John.4.28"
∷ word (γ ∷ υ ∷ ν ∷ ὴ ∷ []) "John.4.28"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.4.28"
∷ word (ἀ ∷ π ∷ ῆ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.4.28"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.4.28"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.4.28"
∷ word (π ∷ ό ∷ ∙λ ∷ ι ∷ ν ∷ []) "John.4.28"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.4.28"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.4.28"
∷ word (τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.4.28"
∷ word (ἀ ∷ ν ∷ θ ∷ ρ ∷ ώ ∷ π ∷ ο ∷ ι ∷ ς ∷ []) "John.4.28"
∷ word (Δ ∷ ε ∷ ῦ ∷ τ ∷ ε ∷ []) "John.4.29"
∷ word (ἴ ∷ δ ∷ ε ∷ τ ∷ ε ∷ []) "John.4.29"
∷ word (ἄ ∷ ν ∷ θ ∷ ρ ∷ ω ∷ π ∷ ο ∷ ν ∷ []) "John.4.29"
∷ word (ὃ ∷ ς ∷ []) "John.4.29"
∷ word (ε ∷ ἶ ∷ π ∷ έ ∷ []) "John.4.29"
∷ word (μ ∷ ο ∷ ι ∷ []) "John.4.29"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ α ∷ []) "John.4.29"
∷ word (ὅ ∷ σ ∷ α ∷ []) "John.4.29"
∷ word (ἐ ∷ π ∷ ο ∷ ί ∷ η ∷ σ ∷ α ∷ []) "John.4.29"
∷ word (μ ∷ ή ∷ τ ∷ ι ∷ []) "John.4.29"
∷ word (ο ∷ ὗ ∷ τ ∷ ό ∷ ς ∷ []) "John.4.29"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.4.29"
∷ word (ὁ ∷ []) "John.4.29"
∷ word (χ ∷ ρ ∷ ι ∷ σ ∷ τ ∷ ό ∷ ς ∷ []) "John.4.29"
∷ word (ἐ ∷ ξ ∷ ῆ ∷ ∙λ ∷ θ ∷ ο ∷ ν ∷ []) "John.4.30"
∷ word (ἐ ∷ κ ∷ []) "John.4.30"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.4.30"
∷ word (π ∷ ό ∷ ∙λ ∷ ε ∷ ω ∷ ς ∷ []) "John.4.30"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.4.30"
∷ word (ἤ ∷ ρ ∷ χ ∷ ο ∷ ν ∷ τ ∷ ο ∷ []) "John.4.30"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.4.30"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.4.30"
∷ word (Ἐ ∷ ν ∷ []) "John.4.31"
∷ word (τ ∷ ῷ ∷ []) "John.4.31"
∷ word (μ ∷ ε ∷ τ ∷ α ∷ ξ ∷ ὺ ∷ []) "John.4.31"
∷ word (ἠ ∷ ρ ∷ ώ ∷ τ ∷ ω ∷ ν ∷ []) "John.4.31"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.4.31"
∷ word (ο ∷ ἱ ∷ []) "John.4.31"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ α ∷ ὶ ∷ []) "John.4.31"
∷ word (∙λ ∷ έ ∷ γ ∷ ο ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.4.31"
∷ word (Ῥ ∷ α ∷ β ∷ β ∷ ί ∷ []) "John.4.31"
∷ word (φ ∷ ά ∷ γ ∷ ε ∷ []) "John.4.31"
∷ word (ὁ ∷ []) "John.4.32"
∷ word (δ ∷ ὲ ∷ []) "John.4.32"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.4.32"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.4.32"
∷ word (Ἐ ∷ γ ∷ ὼ ∷ []) "John.4.32"
∷ word (β ∷ ρ ∷ ῶ ∷ σ ∷ ι ∷ ν ∷ []) "John.4.32"
∷ word (ἔ ∷ χ ∷ ω ∷ []) "John.4.32"
∷ word (φ ∷ α ∷ γ ∷ ε ∷ ῖ ∷ ν ∷ []) "John.4.32"
∷ word (ἣ ∷ ν ∷ []) "John.4.32"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.4.32"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.4.32"
∷ word (ο ∷ ἴ ∷ δ ∷ α ∷ τ ∷ ε ∷ []) "John.4.32"
∷ word (ἔ ∷ ∙λ ∷ ε ∷ γ ∷ ο ∷ ν ∷ []) "John.4.33"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.4.33"
∷ word (ο ∷ ἱ ∷ []) "John.4.33"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ α ∷ ὶ ∷ []) "John.4.33"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.4.33"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ή ∷ ∙λ ∷ ο ∷ υ ∷ ς ∷ []) "John.4.33"
∷ word (Μ ∷ ή ∷ []) "John.4.33"
∷ word (τ ∷ ι ∷ ς ∷ []) "John.4.33"
∷ word (ἤ ∷ ν ∷ ε ∷ γ ∷ κ ∷ ε ∷ ν ∷ []) "John.4.33"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.4.33"
∷ word (φ ∷ α ∷ γ ∷ ε ∷ ῖ ∷ ν ∷ []) "John.4.33"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.4.34"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.4.34"
∷ word (ὁ ∷ []) "John.4.34"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.4.34"
∷ word (Ἐ ∷ μ ∷ ὸ ∷ ν ∷ []) "John.4.34"
∷ word (β ∷ ρ ∷ ῶ ∷ μ ∷ ά ∷ []) "John.4.34"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.4.34"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.4.34"
∷ word (π ∷ ο ∷ ι ∷ ή ∷ σ ∷ ω ∷ []) "John.4.34"
∷ word (τ ∷ ὸ ∷ []) "John.4.34"
∷ word (θ ∷ έ ∷ ∙λ ∷ η ∷ μ ∷ α ∷ []) "John.4.34"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.4.34"
∷ word (π ∷ έ ∷ μ ∷ ψ ∷ α ∷ ν ∷ τ ∷ ό ∷ ς ∷ []) "John.4.34"
∷ word (μ ∷ ε ∷ []) "John.4.34"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.4.34"
∷ word (τ ∷ ε ∷ ∙λ ∷ ε ∷ ι ∷ ώ ∷ σ ∷ ω ∷ []) "John.4.34"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.4.34"
∷ word (τ ∷ ὸ ∷ []) "John.4.34"
∷ word (ἔ ∷ ρ ∷ γ ∷ ο ∷ ν ∷ []) "John.4.34"
∷ word (ο ∷ ὐ ∷ χ ∷ []) "John.4.35"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.4.35"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ τ ∷ ε ∷ []) "John.4.35"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.4.35"
∷ word (Ἔ ∷ τ ∷ ι ∷ []) "John.4.35"
∷ word (τ ∷ ε ∷ τ ∷ ρ ∷ ά ∷ μ ∷ η ∷ ν ∷ ό ∷ ς ∷ []) "John.4.35"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.4.35"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.4.35"
∷ word (ὁ ∷ []) "John.4.35"
∷ word (θ ∷ ε ∷ ρ ∷ ι ∷ σ ∷ μ ∷ ὸ ∷ ς ∷ []) "John.4.35"
∷ word (ἔ ∷ ρ ∷ χ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.4.35"
∷ word (ἰ ∷ δ ∷ ο ∷ ὺ ∷ []) "John.4.35"
∷ word (∙λ ∷ έ ∷ γ ∷ ω ∷ []) "John.4.35"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.4.35"
∷ word (ἐ ∷ π ∷ ά ∷ ρ ∷ α ∷ τ ∷ ε ∷ []) "John.4.35"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.4.35"
∷ word (ὀ ∷ φ ∷ θ ∷ α ∷ ∙λ ∷ μ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.4.35"
∷ word (ὑ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.4.35"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.4.35"
∷ word (θ ∷ ε ∷ ά ∷ σ ∷ α ∷ σ ∷ θ ∷ ε ∷ []) "John.4.35"
∷ word (τ ∷ ὰ ∷ ς ∷ []) "John.4.35"
∷ word (χ ∷ ώ ∷ ρ ∷ α ∷ ς ∷ []) "John.4.35"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.4.35"
∷ word (∙λ ∷ ε ∷ υ ∷ κ ∷ α ∷ ί ∷ []) "John.4.35"
∷ word (ε ∷ ἰ ∷ σ ∷ ι ∷ ν ∷ []) "John.4.35"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.4.35"
∷ word (θ ∷ ε ∷ ρ ∷ ι ∷ σ ∷ μ ∷ ό ∷ ν ∷ []) "John.4.35"
∷ word (ἤ ∷ δ ∷ η ∷ []) "John.4.35"
∷ word (ὁ ∷ []) "John.4.36"
∷ word (θ ∷ ε ∷ ρ ∷ ί ∷ ζ ∷ ω ∷ ν ∷ []) "John.4.36"
∷ word (μ ∷ ι ∷ σ ∷ θ ∷ ὸ ∷ ν ∷ []) "John.4.36"
∷ word (∙λ ∷ α ∷ μ ∷ β ∷ ά ∷ ν ∷ ε ∷ ι ∷ []) "John.4.36"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.4.36"
∷ word (σ ∷ υ ∷ ν ∷ ά ∷ γ ∷ ε ∷ ι ∷ []) "John.4.36"
∷ word (κ ∷ α ∷ ρ ∷ π ∷ ὸ ∷ ν ∷ []) "John.4.36"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.4.36"
∷ word (ζ ∷ ω ∷ ὴ ∷ ν ∷ []) "John.4.36"
∷ word (α ∷ ἰ ∷ ώ ∷ ν ∷ ι ∷ ο ∷ ν ∷ []) "John.4.36"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.4.36"
∷ word (ὁ ∷ []) "John.4.36"
∷ word (σ ∷ π ∷ ε ∷ ί ∷ ρ ∷ ω ∷ ν ∷ []) "John.4.36"
∷ word (ὁ ∷ μ ∷ ο ∷ ῦ ∷ []) "John.4.36"
∷ word (χ ∷ α ∷ ί ∷ ρ ∷ ῃ ∷ []) "John.4.36"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.4.36"
∷ word (ὁ ∷ []) "John.4.36"
∷ word (θ ∷ ε ∷ ρ ∷ ί ∷ ζ ∷ ω ∷ ν ∷ []) "John.4.36"
∷ word (ἐ ∷ ν ∷ []) "John.4.37"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.4.37"
∷ word (τ ∷ ο ∷ ύ ∷ τ ∷ ῳ ∷ []) "John.4.37"
∷ word (ὁ ∷ []) "John.4.37"
∷ word (∙λ ∷ ό ∷ γ ∷ ο ∷ ς ∷ []) "John.4.37"
∷ word (ἐ ∷ σ ∷ τ ∷ ὶ ∷ ν ∷ []) "John.4.37"
∷ word (ἀ ∷ ∙λ ∷ η ∷ θ ∷ ι ∷ ν ∷ ὸ ∷ ς ∷ []) "John.4.37"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.4.37"
∷ word (Ἄ ∷ ∙λ ∷ ∙λ ∷ ο ∷ ς ∷ []) "John.4.37"
∷ word (ἐ ∷ σ ∷ τ ∷ ὶ ∷ ν ∷ []) "John.4.37"
∷ word (ὁ ∷ []) "John.4.37"
∷ word (σ ∷ π ∷ ε ∷ ί ∷ ρ ∷ ω ∷ ν ∷ []) "John.4.37"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.4.37"
∷ word (ἄ ∷ ∙λ ∷ ∙λ ∷ ο ∷ ς ∷ []) "John.4.37"
∷ word (ὁ ∷ []) "John.4.37"
∷ word (θ ∷ ε ∷ ρ ∷ ί ∷ ζ ∷ ω ∷ ν ∷ []) "John.4.37"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.4.38"
∷ word (ἀ ∷ π ∷ έ ∷ σ ∷ τ ∷ ε ∷ ι ∷ ∙λ ∷ α ∷ []) "John.4.38"
∷ word (ὑ ∷ μ ∷ ᾶ ∷ ς ∷ []) "John.4.38"
∷ word (θ ∷ ε ∷ ρ ∷ ί ∷ ζ ∷ ε ∷ ι ∷ ν ∷ []) "John.4.38"
∷ word (ὃ ∷ []) "John.4.38"
∷ word (ο ∷ ὐ ∷ χ ∷ []) "John.4.38"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.4.38"
∷ word (κ ∷ ε ∷ κ ∷ ο ∷ π ∷ ι ∷ ά ∷ κ ∷ α ∷ τ ∷ ε ∷ []) "John.4.38"
∷ word (ἄ ∷ ∙λ ∷ ∙λ ∷ ο ∷ ι ∷ []) "John.4.38"
∷ word (κ ∷ ε ∷ κ ∷ ο ∷ π ∷ ι ∷ ά ∷ κ ∷ α ∷ σ ∷ ι ∷ ν ∷ []) "John.4.38"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.4.38"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.4.38"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.4.38"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.4.38"
∷ word (κ ∷ ό ∷ π ∷ ο ∷ ν ∷ []) "John.4.38"
∷ word (α ∷ ὐ ∷ τ ∷ ῶ ∷ ν ∷ []) "John.4.38"
∷ word (ε ∷ ἰ ∷ σ ∷ ε ∷ ∙λ ∷ η ∷ ∙λ ∷ ύ ∷ θ ∷ α ∷ τ ∷ ε ∷ []) "John.4.38"
∷ word (Ἐ ∷ κ ∷ []) "John.4.39"
∷ word (δ ∷ ὲ ∷ []) "John.4.39"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.4.39"
∷ word (π ∷ ό ∷ ∙λ ∷ ε ∷ ω ∷ ς ∷ []) "John.4.39"
∷ word (ἐ ∷ κ ∷ ε ∷ ί ∷ ν ∷ η ∷ ς ∷ []) "John.4.39"
∷ word (π ∷ ο ∷ ∙λ ∷ ∙λ ∷ ο ∷ ὶ ∷ []) "John.4.39"
∷ word (ἐ ∷ π ∷ ί ∷ σ ∷ τ ∷ ε ∷ υ ∷ σ ∷ α ∷ ν ∷ []) "John.4.39"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.4.39"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.4.39"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.4.39"
∷ word (Σ ∷ α ∷ μ ∷ α ∷ ρ ∷ ι ∷ τ ∷ ῶ ∷ ν ∷ []) "John.4.39"
∷ word (δ ∷ ι ∷ ὰ ∷ []) "John.4.39"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.4.39"
∷ word (∙λ ∷ ό ∷ γ ∷ ο ∷ ν ∷ []) "John.4.39"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.4.39"
∷ word (γ ∷ υ ∷ ν ∷ α ∷ ι ∷ κ ∷ ὸ ∷ ς ∷ []) "John.4.39"
∷ word (μ ∷ α ∷ ρ ∷ τ ∷ υ ∷ ρ ∷ ο ∷ ύ ∷ σ ∷ η ∷ ς ∷ []) "John.4.39"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.4.39"
∷ word (Ε ∷ ἶ ∷ π ∷ έ ∷ ν ∷ []) "John.4.39"
∷ word (μ ∷ ο ∷ ι ∷ []) "John.4.39"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ α ∷ []) "John.4.39"
∷ word (ἃ ∷ []) "John.4.39"
∷ word (ἐ ∷ π ∷ ο ∷ ί ∷ η ∷ σ ∷ α ∷ []) "John.4.39"
∷ word (ὡ ∷ ς ∷ []) "John.4.40"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.4.40"
∷ word (ἦ ∷ ∙λ ∷ θ ∷ ο ∷ ν ∷ []) "John.4.40"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.4.40"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.4.40"
∷ word (ο ∷ ἱ ∷ []) "John.4.40"
∷ word (Σ ∷ α ∷ μ ∷ α ∷ ρ ∷ ῖ ∷ τ ∷ α ∷ ι ∷ []) "John.4.40"
∷ word (ἠ ∷ ρ ∷ ώ ∷ τ ∷ ω ∷ ν ∷ []) "John.4.40"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.4.40"
∷ word (μ ∷ ε ∷ ῖ ∷ ν ∷ α ∷ ι ∷ []) "John.4.40"
∷ word (π ∷ α ∷ ρ ∷ []) "John.4.40"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.4.40"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.4.40"
∷ word (ἔ ∷ μ ∷ ε ∷ ι ∷ ν ∷ ε ∷ ν ∷ []) "John.4.40"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ []) "John.4.40"
∷ word (δ ∷ ύ ∷ ο ∷ []) "John.4.40"
∷ word (ἡ ∷ μ ∷ έ ∷ ρ ∷ α ∷ ς ∷ []) "John.4.40"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.4.41"
∷ word (π ∷ ο ∷ ∙λ ∷ ∙λ ∷ ῷ ∷ []) "John.4.41"
∷ word (π ∷ ∙λ ∷ ε ∷ ί ∷ ο ∷ υ ∷ ς ∷ []) "John.4.41"
∷ word (ἐ ∷ π ∷ ί ∷ σ ∷ τ ∷ ε ∷ υ ∷ σ ∷ α ∷ ν ∷ []) "John.4.41"
∷ word (δ ∷ ι ∷ ὰ ∷ []) "John.4.41"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.4.41"
∷ word (∙λ ∷ ό ∷ γ ∷ ο ∷ ν ∷ []) "John.4.41"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.4.41"
∷ word (τ ∷ ῇ ∷ []) "John.4.42"
∷ word (τ ∷ ε ∷ []) "John.4.42"
∷ word (γ ∷ υ ∷ ν ∷ α ∷ ι ∷ κ ∷ ὶ ∷ []) "John.4.42"
∷ word (ἔ ∷ ∙λ ∷ ε ∷ γ ∷ ο ∷ ν ∷ []) "John.4.42"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.4.42"
∷ word (Ο ∷ ὐ ∷ κ ∷ έ ∷ τ ∷ ι ∷ []) "John.4.42"
∷ word (δ ∷ ι ∷ ὰ ∷ []) "John.4.42"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.4.42"
∷ word (σ ∷ ὴ ∷ ν ∷ []) "John.4.42"
∷ word (∙λ ∷ α ∷ ∙λ ∷ ι ∷ ὰ ∷ ν ∷ []) "John.4.42"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ ο ∷ μ ∷ ε ∷ ν ∷ []) "John.4.42"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ὶ ∷ []) "John.4.42"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.4.42"
∷ word (ἀ ∷ κ ∷ η ∷ κ ∷ ό ∷ α ∷ μ ∷ ε ∷ ν ∷ []) "John.4.42"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.4.42"
∷ word (ο ∷ ἴ ∷ δ ∷ α ∷ μ ∷ ε ∷ ν ∷ []) "John.4.42"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.4.42"
∷ word (ο ∷ ὗ ∷ τ ∷ ό ∷ ς ∷ []) "John.4.42"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.4.42"
∷ word (ἀ ∷ ∙λ ∷ η ∷ θ ∷ ῶ ∷ ς ∷ []) "John.4.42"
∷ word (ὁ ∷ []) "John.4.42"
∷ word (σ ∷ ω ∷ τ ∷ ὴ ∷ ρ ∷ []) "John.4.42"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.4.42"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ υ ∷ []) "John.4.42"
∷ word (Μ ∷ ε ∷ τ ∷ ὰ ∷ []) "John.4.43"
∷ word (δ ∷ ὲ ∷ []) "John.4.43"
∷ word (τ ∷ ὰ ∷ ς ∷ []) "John.4.43"
∷ word (δ ∷ ύ ∷ ο ∷ []) "John.4.43"
∷ word (ἡ ∷ μ ∷ έ ∷ ρ ∷ α ∷ ς ∷ []) "John.4.43"
∷ word (ἐ ∷ ξ ∷ ῆ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.4.43"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ θ ∷ ε ∷ ν ∷ []) "John.4.43"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.4.43"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.4.43"
∷ word (Γ ∷ α ∷ ∙λ ∷ ι ∷ ∙λ ∷ α ∷ ί ∷ α ∷ ν ∷ []) "John.4.43"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ς ∷ []) "John.4.44"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.4.44"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.4.44"
∷ word (ἐ ∷ μ ∷ α ∷ ρ ∷ τ ∷ ύ ∷ ρ ∷ η ∷ σ ∷ ε ∷ ν ∷ []) "John.4.44"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.4.44"
∷ word (π ∷ ρ ∷ ο ∷ φ ∷ ή ∷ τ ∷ η ∷ ς ∷ []) "John.4.44"
∷ word (ἐ ∷ ν ∷ []) "John.4.44"
∷ word (τ ∷ ῇ ∷ []) "John.4.44"
∷ word (ἰ ∷ δ ∷ ί ∷ ᾳ ∷ []) "John.4.44"
∷ word (π ∷ α ∷ τ ∷ ρ ∷ ί ∷ δ ∷ ι ∷ []) "John.4.44"
∷ word (τ ∷ ι ∷ μ ∷ ὴ ∷ ν ∷ []) "John.4.44"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.4.44"
∷ word (ἔ ∷ χ ∷ ε ∷ ι ∷ []) "John.4.44"
∷ word (ὅ ∷ τ ∷ ε ∷ []) "John.4.45"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.4.45"
∷ word (ἦ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.4.45"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.4.45"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.4.45"
∷ word (Γ ∷ α ∷ ∙λ ∷ ι ∷ ∙λ ∷ α ∷ ί ∷ α ∷ ν ∷ []) "John.4.45"
∷ word (ἐ ∷ δ ∷ έ ∷ ξ ∷ α ∷ ν ∷ τ ∷ ο ∷ []) "John.4.45"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.4.45"
∷ word (ο ∷ ἱ ∷ []) "John.4.45"
∷ word (Γ ∷ α ∷ ∙λ ∷ ι ∷ ∙λ ∷ α ∷ ῖ ∷ ο ∷ ι ∷ []) "John.4.45"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ α ∷ []) "John.4.45"
∷ word (ἑ ∷ ω ∷ ρ ∷ α ∷ κ ∷ ό ∷ τ ∷ ε ∷ ς ∷ []) "John.4.45"
∷ word (ὅ ∷ σ ∷ α ∷ []) "John.4.45"
∷ word (ἐ ∷ π ∷ ο ∷ ί ∷ η ∷ σ ∷ ε ∷ ν ∷ []) "John.4.45"
∷ word (ἐ ∷ ν ∷ []) "John.4.45"
∷ word (Ἱ ∷ ε ∷ ρ ∷ ο ∷ σ ∷ ο ∷ ∙λ ∷ ύ ∷ μ ∷ ο ∷ ι ∷ ς ∷ []) "John.4.45"
∷ word (ἐ ∷ ν ∷ []) "John.4.45"
∷ word (τ ∷ ῇ ∷ []) "John.4.45"
∷ word (ἑ ∷ ο ∷ ρ ∷ τ ∷ ῇ ∷ []) "John.4.45"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.4.45"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ὶ ∷ []) "John.4.45"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.4.45"
∷ word (ἦ ∷ ∙λ ∷ θ ∷ ο ∷ ν ∷ []) "John.4.45"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.4.45"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.4.45"
∷ word (ἑ ∷ ο ∷ ρ ∷ τ ∷ ή ∷ ν ∷ []) "John.4.45"
∷ word (Ἦ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.4.46"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.4.46"
∷ word (π ∷ ά ∷ ∙λ ∷ ι ∷ ν ∷ []) "John.4.46"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.4.46"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.4.46"
∷ word (Κ ∷ α ∷ ν ∷ ὰ ∷ []) "John.4.46"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.4.46"
∷ word (Γ ∷ α ∷ ∙λ ∷ ι ∷ ∙λ ∷ α ∷ ί ∷ α ∷ ς ∷ []) "John.4.46"
∷ word (ὅ ∷ π ∷ ο ∷ υ ∷ []) "John.4.46"
∷ word (ἐ ∷ π ∷ ο ∷ ί ∷ η ∷ σ ∷ ε ∷ ν ∷ []) "John.4.46"
∷ word (τ ∷ ὸ ∷ []) "John.4.46"
∷ word (ὕ ∷ δ ∷ ω ∷ ρ ∷ []) "John.4.46"
∷ word (ο ∷ ἶ ∷ ν ∷ ο ∷ ν ∷ []) "John.4.46"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.4.46"
∷ word (ἦ ∷ ν ∷ []) "John.4.46"
∷ word (τ ∷ ι ∷ ς ∷ []) "John.4.46"
∷ word (β ∷ α ∷ σ ∷ ι ∷ ∙λ ∷ ι ∷ κ ∷ ὸ ∷ ς ∷ []) "John.4.46"
∷ word (ο ∷ ὗ ∷ []) "John.4.46"
∷ word (ὁ ∷ []) "John.4.46"
∷ word (υ ∷ ἱ ∷ ὸ ∷ ς ∷ []) "John.4.46"
∷ word (ἠ ∷ σ ∷ θ ∷ έ ∷ ν ∷ ε ∷ ι ∷ []) "John.4.46"
∷ word (ἐ ∷ ν ∷ []) "John.4.46"
∷ word (Κ ∷ α ∷ φ ∷ α ∷ ρ ∷ ν ∷ α ∷ ο ∷ ύ ∷ μ ∷ []) "John.4.46"
∷ word (ο ∷ ὗ ∷ τ ∷ ο ∷ ς ∷ []) "John.4.47"
∷ word (ἀ ∷ κ ∷ ο ∷ ύ ∷ σ ∷ α ∷ ς ∷ []) "John.4.47"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.4.47"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.4.47"
∷ word (ἥ ∷ κ ∷ ε ∷ ι ∷ []) "John.4.47"
∷ word (ἐ ∷ κ ∷ []) "John.4.47"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.4.47"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ί ∷ α ∷ ς ∷ []) "John.4.47"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.4.47"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.4.47"
∷ word (Γ ∷ α ∷ ∙λ ∷ ι ∷ ∙λ ∷ α ∷ ί ∷ α ∷ ν ∷ []) "John.4.47"
∷ word (ἀ ∷ π ∷ ῆ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.4.47"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.4.47"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.4.47"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.4.47"
∷ word (ἠ ∷ ρ ∷ ώ ∷ τ ∷ α ∷ []) "John.4.47"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.4.47"
∷ word (κ ∷ α ∷ τ ∷ α ∷ β ∷ ῇ ∷ []) "John.4.47"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.4.47"
∷ word (ἰ ∷ ά ∷ σ ∷ η ∷ τ ∷ α ∷ ι ∷ []) "John.4.47"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.4.47"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.4.47"
∷ word (υ ∷ ἱ ∷ ό ∷ ν ∷ []) "John.4.47"
∷ word (ἤ ∷ μ ∷ ε ∷ ∙λ ∷ ∙λ ∷ ε ∷ ν ∷ []) "John.4.47"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.4.47"
∷ word (ἀ ∷ π ∷ ο ∷ θ ∷ ν ∷ ῄ ∷ σ ∷ κ ∷ ε ∷ ι ∷ ν ∷ []) "John.4.47"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.4.48"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.4.48"
∷ word (ὁ ∷ []) "John.4.48"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.4.48"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.4.48"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.4.48"
∷ word (Ἐ ∷ ὰ ∷ ν ∷ []) "John.4.48"
∷ word (μ ∷ ὴ ∷ []) "John.4.48"
∷ word (σ ∷ η ∷ μ ∷ ε ∷ ῖ ∷ α ∷ []) "John.4.48"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.4.48"
∷ word (τ ∷ έ ∷ ρ ∷ α ∷ τ ∷ α ∷ []) "John.4.48"
∷ word (ἴ ∷ δ ∷ η ∷ τ ∷ ε ∷ []) "John.4.48"
∷ word (ο ∷ ὐ ∷ []) "John.4.48"
∷ word (μ ∷ ὴ ∷ []) "John.4.48"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ σ ∷ η ∷ τ ∷ ε ∷ []) "John.4.48"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.4.49"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.4.49"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.4.49"
∷ word (ὁ ∷ []) "John.4.49"
∷ word (β ∷ α ∷ σ ∷ ι ∷ ∙λ ∷ ι ∷ κ ∷ ό ∷ ς ∷ []) "John.4.49"
∷ word (Κ ∷ ύ ∷ ρ ∷ ι ∷ ε ∷ []) "John.4.49"
∷ word (κ ∷ α ∷ τ ∷ ά ∷ β ∷ η ∷ θ ∷ ι ∷ []) "John.4.49"
∷ word (π ∷ ρ ∷ ὶ ∷ ν ∷ []) "John.4.49"
∷ word (ἀ ∷ π ∷ ο ∷ θ ∷ α ∷ ν ∷ ε ∷ ῖ ∷ ν ∷ []) "John.4.49"
∷ word (τ ∷ ὸ ∷ []) "John.4.49"
∷ word (π ∷ α ∷ ι ∷ δ ∷ ί ∷ ο ∷ ν ∷ []) "John.4.49"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.4.49"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.4.50"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.4.50"
∷ word (ὁ ∷ []) "John.4.50"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.4.50"
∷ word (Π ∷ ο ∷ ρ ∷ ε ∷ ύ ∷ ο ∷ υ ∷ []) "John.4.50"
∷ word (ὁ ∷ []) "John.4.50"
∷ word (υ ∷ ἱ ∷ ό ∷ ς ∷ []) "John.4.50"
∷ word (σ ∷ ο ∷ υ ∷ []) "John.4.50"
∷ word (ζ ∷ ῇ ∷ []) "John.4.50"
∷ word (ἐ ∷ π ∷ ί ∷ σ ∷ τ ∷ ε ∷ υ ∷ σ ∷ ε ∷ ν ∷ []) "John.4.50"
∷ word (ὁ ∷ []) "John.4.50"
∷ word (ἄ ∷ ν ∷ θ ∷ ρ ∷ ω ∷ π ∷ ο ∷ ς ∷ []) "John.4.50"
∷ word (τ ∷ ῷ ∷ []) "John.4.50"
∷ word (∙λ ∷ ό ∷ γ ∷ ῳ ∷ []) "John.4.50"
∷ word (ὃ ∷ ν ∷ []) "John.4.50"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.4.50"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.4.50"
∷ word (ὁ ∷ []) "John.4.50"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.4.50"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.4.50"
∷ word (ἐ ∷ π ∷ ο ∷ ρ ∷ ε ∷ ύ ∷ ε ∷ τ ∷ ο ∷ []) "John.4.50"
∷ word (ἤ ∷ δ ∷ η ∷ []) "John.4.51"
∷ word (δ ∷ ὲ ∷ []) "John.4.51"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.4.51"
∷ word (κ ∷ α ∷ τ ∷ α ∷ β ∷ α ∷ ί ∷ ν ∷ ο ∷ ν ∷ τ ∷ ο ∷ ς ∷ []) "John.4.51"
∷ word (ο ∷ ἱ ∷ []) "John.4.51"
∷ word (δ ∷ ο ∷ ῦ ∷ ∙λ ∷ ο ∷ ι ∷ []) "John.4.51"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.4.51"
∷ word (ὑ ∷ π ∷ ή ∷ ν ∷ τ ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.4.51"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.4.51"
∷ word (∙λ ∷ έ ∷ γ ∷ ο ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.4.51"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.4.51"
∷ word (ὁ ∷ []) "John.4.51"
∷ word (π ∷ α ∷ ῖ ∷ ς ∷ []) "John.4.51"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.4.51"
∷ word (ζ ∷ ῇ ∷ []) "John.4.51"
∷ word (ἐ ∷ π ∷ ύ ∷ θ ∷ ε ∷ τ ∷ ο ∷ []) "John.4.52"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.4.52"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.4.52"
∷ word (ὥ ∷ ρ ∷ α ∷ ν ∷ []) "John.4.52"
∷ word (π ∷ α ∷ ρ ∷ []) "John.4.52"
∷ word (α ∷ ὐ ∷ τ ∷ ῶ ∷ ν ∷ []) "John.4.52"
∷ word (ἐ ∷ ν ∷ []) "John.4.52"
∷ word (ᾗ ∷ []) "John.4.52"
∷ word (κ ∷ ο ∷ μ ∷ ψ ∷ ό ∷ τ ∷ ε ∷ ρ ∷ ο ∷ ν ∷ []) "John.4.52"
∷ word (ἔ ∷ σ ∷ χ ∷ ε ∷ ν ∷ []) "John.4.52"
∷ word (ε ∷ ἶ ∷ π ∷ α ∷ ν ∷ []) "John.4.52"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.4.52"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.4.52"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.4.52"
∷ word (Ἐ ∷ χ ∷ θ ∷ ὲ ∷ ς ∷ []) "John.4.52"
∷ word (ὥ ∷ ρ ∷ α ∷ ν ∷ []) "John.4.52"
∷ word (ἑ ∷ β ∷ δ ∷ ό ∷ μ ∷ η ∷ ν ∷ []) "John.4.52"
∷ word (ἀ ∷ φ ∷ ῆ ∷ κ ∷ ε ∷ ν ∷ []) "John.4.52"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.4.52"
∷ word (ὁ ∷ []) "John.4.52"
∷ word (π ∷ υ ∷ ρ ∷ ε ∷ τ ∷ ό ∷ ς ∷ []) "John.4.52"
∷ word (ἔ ∷ γ ∷ ν ∷ ω ∷ []) "John.4.53"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.4.53"
∷ word (ὁ ∷ []) "John.4.53"
∷ word (π ∷ α ∷ τ ∷ ὴ ∷ ρ ∷ []) "John.4.53"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.4.53"
∷ word (ἐ ∷ κ ∷ ε ∷ ί ∷ ν ∷ ῃ ∷ []) "John.4.53"
∷ word (τ ∷ ῇ ∷ []) "John.4.53"
∷ word (ὥ ∷ ρ ∷ ᾳ ∷ []) "John.4.53"
∷ word (ἐ ∷ ν ∷ []) "John.4.53"
∷ word (ᾗ ∷ []) "John.4.53"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.4.53"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.4.53"
∷ word (ὁ ∷ []) "John.4.53"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.4.53"
∷ word (Ὁ ∷ []) "John.4.53"
∷ word (υ ∷ ἱ ∷ ό ∷ ς ∷ []) "John.4.53"
∷ word (σ ∷ ο ∷ υ ∷ []) "John.4.53"
∷ word (ζ ∷ ῇ ∷ []) "John.4.53"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.4.53"
∷ word (ἐ ∷ π ∷ ί ∷ σ ∷ τ ∷ ε ∷ υ ∷ σ ∷ ε ∷ ν ∷ []) "John.4.53"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ς ∷ []) "John.4.53"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.4.53"
∷ word (ἡ ∷ []) "John.4.53"
∷ word (ο ∷ ἰ ∷ κ ∷ ί ∷ α ∷ []) "John.4.53"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.4.53"
∷ word (ὅ ∷ ∙λ ∷ η ∷ []) "John.4.53"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.4.54"
∷ word (δ ∷ ὲ ∷ []) "John.4.54"
∷ word (π ∷ ά ∷ ∙λ ∷ ι ∷ ν ∷ []) "John.4.54"
∷ word (δ ∷ ε ∷ ύ ∷ τ ∷ ε ∷ ρ ∷ ο ∷ ν ∷ []) "John.4.54"
∷ word (σ ∷ η ∷ μ ∷ ε ∷ ῖ ∷ ο ∷ ν ∷ []) "John.4.54"
∷ word (ἐ ∷ π ∷ ο ∷ ί ∷ η ∷ σ ∷ ε ∷ ν ∷ []) "John.4.54"
∷ word (ὁ ∷ []) "John.4.54"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.4.54"
∷ word (ἐ ∷ ∙λ ∷ θ ∷ ὼ ∷ ν ∷ []) "John.4.54"
∷ word (ἐ ∷ κ ∷ []) "John.4.54"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.4.54"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ί ∷ α ∷ ς ∷ []) "John.4.54"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.4.54"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.4.54"
∷ word (Γ ∷ α ∷ ∙λ ∷ ι ∷ ∙λ ∷ α ∷ ί ∷ α ∷ ν ∷ []) "John.4.54"
∷ word (Μ ∷ ε ∷ τ ∷ ὰ ∷ []) "John.5.1"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.5.1"
∷ word (ἦ ∷ ν ∷ []) "John.5.1"
∷ word (ἑ ∷ ο ∷ ρ ∷ τ ∷ ὴ ∷ []) "John.5.1"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.5.1"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ί ∷ ω ∷ ν ∷ []) "John.5.1"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.5.1"
∷ word (ἀ ∷ ν ∷ έ ∷ β ∷ η ∷ []) "John.5.1"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.5.1"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.5.1"
∷ word (Ἱ ∷ ε ∷ ρ ∷ ο ∷ σ ∷ ό ∷ ∙λ ∷ υ ∷ μ ∷ α ∷ []) "John.5.1"
∷ word (ἔ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.5.2"
∷ word (δ ∷ ὲ ∷ []) "John.5.2"
∷ word (ἐ ∷ ν ∷ []) "John.5.2"
∷ word (τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.5.2"
∷ word (Ἱ ∷ ε ∷ ρ ∷ ο ∷ σ ∷ ο ∷ ∙λ ∷ ύ ∷ μ ∷ ο ∷ ι ∷ ς ∷ []) "John.5.2"
∷ word (ἐ ∷ π ∷ ὶ ∷ []) "John.5.2"
∷ word (τ ∷ ῇ ∷ []) "John.5.2"
∷ word (π ∷ ρ ∷ ο ∷ β ∷ α ∷ τ ∷ ι ∷ κ ∷ ῇ ∷ []) "John.5.2"
∷ word (κ ∷ ο ∷ ∙λ ∷ υ ∷ μ ∷ β ∷ ή ∷ θ ∷ ρ ∷ α ∷ []) "John.5.2"
∷ word (ἡ ∷ []) "John.5.2"
∷ word (ἐ ∷ π ∷ ι ∷ ∙λ ∷ ε ∷ γ ∷ ο ∷ μ ∷ έ ∷ ν ∷ η ∷ []) "John.5.2"
∷ word (Ἑ ∷ β ∷ ρ ∷ α ∷ ϊ ∷ σ ∷ τ ∷ ὶ ∷ []) "John.5.2"
∷ word (Β ∷ η ∷ θ ∷ ε ∷ σ ∷ δ ∷ ά ∷ []) "John.5.2"
∷ word (π ∷ έ ∷ ν ∷ τ ∷ ε ∷ []) "John.5.2"
∷ word (σ ∷ τ ∷ ο ∷ ὰ ∷ ς ∷ []) "John.5.2"
∷ word (ἔ ∷ χ ∷ ο ∷ υ ∷ σ ∷ α ∷ []) "John.5.2"
∷ word (ἐ ∷ ν ∷ []) "John.5.3"
∷ word (τ ∷ α ∷ ύ ∷ τ ∷ α ∷ ι ∷ ς ∷ []) "John.5.3"
∷ word (κ ∷ α ∷ τ ∷ έ ∷ κ ∷ ε ∷ ι ∷ τ ∷ ο ∷ []) "John.5.3"
∷ word (π ∷ ∙λ ∷ ῆ ∷ θ ∷ ο ∷ ς ∷ []) "John.5.3"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.5.3"
∷ word (ἀ ∷ σ ∷ θ ∷ ε ∷ ν ∷ ο ∷ ύ ∷ ν ∷ τ ∷ ω ∷ ν ∷ []) "John.5.3"
∷ word (τ ∷ υ ∷ φ ∷ ∙λ ∷ ῶ ∷ ν ∷ []) "John.5.3"
∷ word (χ ∷ ω ∷ ∙λ ∷ ῶ ∷ ν ∷ []) "John.5.3"
∷ word (ξ ∷ η ∷ ρ ∷ ῶ ∷ ν ∷ []) "John.5.3"
∷ word (ἦ ∷ ν ∷ []) "John.5.5"
∷ word (δ ∷ έ ∷ []) "John.5.5"
∷ word (τ ∷ ι ∷ ς ∷ []) "John.5.5"
∷ word (ἄ ∷ ν ∷ θ ∷ ρ ∷ ω ∷ π ∷ ο ∷ ς ∷ []) "John.5.5"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ []) "John.5.5"
∷ word (τ ∷ ρ ∷ ι ∷ ά ∷ κ ∷ ο ∷ ν ∷ τ ∷ α ∷ []) "John.5.5"
∷ word (ὀ ∷ κ ∷ τ ∷ ὼ ∷ []) "John.5.5"
∷ word (ἔ ∷ τ ∷ η ∷ []) "John.5.5"
∷ word (ἔ ∷ χ ∷ ω ∷ ν ∷ []) "John.5.5"
∷ word (ἐ ∷ ν ∷ []) "John.5.5"
∷ word (τ ∷ ῇ ∷ []) "John.5.5"
∷ word (ἀ ∷ σ ∷ θ ∷ ε ∷ ν ∷ ε ∷ ί ∷ ᾳ ∷ []) "John.5.5"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.5.5"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ ν ∷ []) "John.5.6"
∷ word (ἰ ∷ δ ∷ ὼ ∷ ν ∷ []) "John.5.6"
∷ word (ὁ ∷ []) "John.5.6"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.5.6"
∷ word (κ ∷ α ∷ τ ∷ α ∷ κ ∷ ε ∷ ί ∷ μ ∷ ε ∷ ν ∷ ο ∷ ν ∷ []) "John.5.6"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.5.6"
∷ word (γ ∷ ν ∷ ο ∷ ὺ ∷ ς ∷ []) "John.5.6"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.5.6"
∷ word (π ∷ ο ∷ ∙λ ∷ ὺ ∷ ν ∷ []) "John.5.6"
∷ word (ἤ ∷ δ ∷ η ∷ []) "John.5.6"
∷ word (χ ∷ ρ ∷ ό ∷ ν ∷ ο ∷ ν ∷ []) "John.5.6"
∷ word (ἔ ∷ χ ∷ ε ∷ ι ∷ []) "John.5.6"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.5.6"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.5.6"
∷ word (Θ ∷ έ ∷ ∙λ ∷ ε ∷ ι ∷ ς ∷ []) "John.5.6"
∷ word (ὑ ∷ γ ∷ ι ∷ ὴ ∷ ς ∷ []) "John.5.6"
∷ word (γ ∷ ε ∷ ν ∷ έ ∷ σ ∷ θ ∷ α ∷ ι ∷ []) "John.5.6"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.5.7"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.5.7"
∷ word (ὁ ∷ []) "John.5.7"
∷ word (ἀ ∷ σ ∷ θ ∷ ε ∷ ν ∷ ῶ ∷ ν ∷ []) "John.5.7"
∷ word (Κ ∷ ύ ∷ ρ ∷ ι ∷ ε ∷ []) "John.5.7"
∷ word (ἄ ∷ ν ∷ θ ∷ ρ ∷ ω ∷ π ∷ ο ∷ ν ∷ []) "John.5.7"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.5.7"
∷ word (ἔ ∷ χ ∷ ω ∷ []) "John.5.7"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.5.7"
∷ word (ὅ ∷ τ ∷ α ∷ ν ∷ []) "John.5.7"
∷ word (τ ∷ α ∷ ρ ∷ α ∷ χ ∷ θ ∷ ῇ ∷ []) "John.5.7"
∷ word (τ ∷ ὸ ∷ []) "John.5.7"
∷ word (ὕ ∷ δ ∷ ω ∷ ρ ∷ []) "John.5.7"
∷ word (β ∷ ά ∷ ∙λ ∷ ῃ ∷ []) "John.5.7"
∷ word (μ ∷ ε ∷ []) "John.5.7"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.5.7"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.5.7"
∷ word (κ ∷ ο ∷ ∙λ ∷ υ ∷ μ ∷ β ∷ ή ∷ θ ∷ ρ ∷ α ∷ ν ∷ []) "John.5.7"
∷ word (ἐ ∷ ν ∷ []) "John.5.7"
∷ word (ᾧ ∷ []) "John.5.7"
∷ word (δ ∷ ὲ ∷ []) "John.5.7"
∷ word (ἔ ∷ ρ ∷ χ ∷ ο ∷ μ ∷ α ∷ ι ∷ []) "John.5.7"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.5.7"
∷ word (ἄ ∷ ∙λ ∷ ∙λ ∷ ο ∷ ς ∷ []) "John.5.7"
∷ word (π ∷ ρ ∷ ὸ ∷ []) "John.5.7"
∷ word (ἐ ∷ μ ∷ ο ∷ ῦ ∷ []) "John.5.7"
∷ word (κ ∷ α ∷ τ ∷ α ∷ β ∷ α ∷ ί ∷ ν ∷ ε ∷ ι ∷ []) "John.5.7"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.5.8"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.5.8"
∷ word (ὁ ∷ []) "John.5.8"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.5.8"
∷ word (Ἔ ∷ γ ∷ ε ∷ ι ∷ ρ ∷ ε ∷ []) "John.5.8"
∷ word (ἆ ∷ ρ ∷ ο ∷ ν ∷ []) "John.5.8"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.5.8"
∷ word (κ ∷ ρ ∷ ά ∷ β ∷ α ∷ τ ∷ τ ∷ ό ∷ ν ∷ []) "John.5.8"
∷ word (σ ∷ ο ∷ υ ∷ []) "John.5.8"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.5.8"
∷ word (π ∷ ε ∷ ρ ∷ ι ∷ π ∷ ά ∷ τ ∷ ε ∷ ι ∷ []) "John.5.8"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.5.9"
∷ word (ε ∷ ὐ ∷ θ ∷ έ ∷ ω ∷ ς ∷ []) "John.5.9"
∷ word (ἐ ∷ γ ∷ έ ∷ ν ∷ ε ∷ τ ∷ ο ∷ []) "John.5.9"
∷ word (ὑ ∷ γ ∷ ι ∷ ὴ ∷ ς ∷ []) "John.5.9"
∷ word (ὁ ∷ []) "John.5.9"
∷ word (ἄ ∷ ν ∷ θ ∷ ρ ∷ ω ∷ π ∷ ο ∷ ς ∷ []) "John.5.9"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.5.9"
∷ word (ἦ ∷ ρ ∷ ε ∷ []) "John.5.9"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.5.9"
∷ word (κ ∷ ρ ∷ ά ∷ β ∷ α ∷ τ ∷ τ ∷ ο ∷ ν ∷ []) "John.5.9"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.5.9"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.5.9"
∷ word (π ∷ ε ∷ ρ ∷ ι ∷ ε ∷ π ∷ ά ∷ τ ∷ ε ∷ ι ∷ []) "John.5.9"
∷ word (Ἦ ∷ ν ∷ []) "John.5.9"
∷ word (δ ∷ ὲ ∷ []) "John.5.9"
∷ word (σ ∷ ά ∷ β ∷ β ∷ α ∷ τ ∷ ο ∷ ν ∷ []) "John.5.9"
∷ word (ἐ ∷ ν ∷ []) "John.5.9"
∷ word (ἐ ∷ κ ∷ ε ∷ ί ∷ ν ∷ ῃ ∷ []) "John.5.9"
∷ word (τ ∷ ῇ ∷ []) "John.5.9"
∷ word (ἡ ∷ μ ∷ έ ∷ ρ ∷ ᾳ ∷ []) "John.5.9"
∷ word (ἔ ∷ ∙λ ∷ ε ∷ γ ∷ ο ∷ ν ∷ []) "John.5.10"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.5.10"
∷ word (ο ∷ ἱ ∷ []) "John.5.10"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ῖ ∷ ο ∷ ι ∷ []) "John.5.10"
∷ word (τ ∷ ῷ ∷ []) "John.5.10"
∷ word (τ ∷ ε ∷ θ ∷ ε ∷ ρ ∷ α ∷ π ∷ ε ∷ υ ∷ μ ∷ έ ∷ ν ∷ ῳ ∷ []) "John.5.10"
∷ word (Σ ∷ ά ∷ β ∷ β ∷ α ∷ τ ∷ ό ∷ ν ∷ []) "John.5.10"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.5.10"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.5.10"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.5.10"
∷ word (ἔ ∷ ξ ∷ ε ∷ σ ∷ τ ∷ ί ∷ ν ∷ []) "John.5.10"
∷ word (σ ∷ ο ∷ ι ∷ []) "John.5.10"
∷ word (ἆ ∷ ρ ∷ α ∷ ι ∷ []) "John.5.10"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.5.10"
∷ word (κ ∷ ρ ∷ ά ∷ β ∷ α ∷ τ ∷ τ ∷ ο ∷ ν ∷ []) "John.5.10"
∷ word (ὃ ∷ ς ∷ []) "John.5.11"
∷ word (δ ∷ ὲ ∷ []) "John.5.11"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.5.11"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.5.11"
∷ word (Ὁ ∷ []) "John.5.11"
∷ word (π ∷ ο ∷ ι ∷ ή ∷ σ ∷ α ∷ ς ∷ []) "John.5.11"
∷ word (μ ∷ ε ∷ []) "John.5.11"
∷ word (ὑ ∷ γ ∷ ι ∷ ῆ ∷ []) "John.5.11"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ό ∷ ς ∷ []) "John.5.11"
∷ word (μ ∷ ο ∷ ι ∷ []) "John.5.11"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.5.11"
∷ word (Ἆ ∷ ρ ∷ ο ∷ ν ∷ []) "John.5.11"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.5.11"
∷ word (κ ∷ ρ ∷ ά ∷ β ∷ α ∷ τ ∷ τ ∷ ό ∷ ν ∷ []) "John.5.11"
∷ word (σ ∷ ο ∷ υ ∷ []) "John.5.11"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.5.11"
∷ word (π ∷ ε ∷ ρ ∷ ι ∷ π ∷ ά ∷ τ ∷ ε ∷ ι ∷ []) "John.5.11"
∷ word (ἠ ∷ ρ ∷ ώ ∷ τ ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.5.12"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.5.12"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.5.12"
∷ word (Τ ∷ ί ∷ ς ∷ []) "John.5.12"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.5.12"
∷ word (ὁ ∷ []) "John.5.12"
∷ word (ἄ ∷ ν ∷ θ ∷ ρ ∷ ω ∷ π ∷ ο ∷ ς ∷ []) "John.5.12"
∷ word (ὁ ∷ []) "John.5.12"
∷ word (ε ∷ ἰ ∷ π ∷ ώ ∷ ν ∷ []) "John.5.12"
∷ word (σ ∷ ο ∷ ι ∷ []) "John.5.12"
∷ word (Ἆ ∷ ρ ∷ ο ∷ ν ∷ []) "John.5.12"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.5.12"
∷ word (π ∷ ε ∷ ρ ∷ ι ∷ π ∷ ά ∷ τ ∷ ε ∷ ι ∷ []) "John.5.12"
∷ word (ὁ ∷ []) "John.5.13"
∷ word (δ ∷ ὲ ∷ []) "John.5.13"
∷ word (ἰ ∷ α ∷ θ ∷ ε ∷ ὶ ∷ ς ∷ []) "John.5.13"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.5.13"
∷ word (ᾔ ∷ δ ∷ ε ∷ ι ∷ []) "John.5.13"
∷ word (τ ∷ ί ∷ ς ∷ []) "John.5.13"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.5.13"
∷ word (ὁ ∷ []) "John.5.13"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.5.13"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.5.13"
∷ word (ἐ ∷ ξ ∷ έ ∷ ν ∷ ε ∷ υ ∷ σ ∷ ε ∷ ν ∷ []) "John.5.13"
∷ word (ὄ ∷ χ ∷ ∙λ ∷ ο ∷ υ ∷ []) "John.5.13"
∷ word (ὄ ∷ ν ∷ τ ∷ ο ∷ ς ∷ []) "John.5.13"
∷ word (ἐ ∷ ν ∷ []) "John.5.13"
∷ word (τ ∷ ῷ ∷ []) "John.5.13"
∷ word (τ ∷ ό ∷ π ∷ ῳ ∷ []) "John.5.13"
∷ word (μ ∷ ε ∷ τ ∷ ὰ ∷ []) "John.5.14"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.5.14"
∷ word (ε ∷ ὑ ∷ ρ ∷ ί ∷ σ ∷ κ ∷ ε ∷ ι ∷ []) "John.5.14"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.5.14"
∷ word (ὁ ∷ []) "John.5.14"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.5.14"
∷ word (ἐ ∷ ν ∷ []) "John.5.14"
∷ word (τ ∷ ῷ ∷ []) "John.5.14"
∷ word (ἱ ∷ ε ∷ ρ ∷ ῷ ∷ []) "John.5.14"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.5.14"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.5.14"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.5.14"
∷ word (Ἴ ∷ δ ∷ ε ∷ []) "John.5.14"
∷ word (ὑ ∷ γ ∷ ι ∷ ὴ ∷ ς ∷ []) "John.5.14"
∷ word (γ ∷ έ ∷ γ ∷ ο ∷ ν ∷ α ∷ ς ∷ []) "John.5.14"
∷ word (μ ∷ η ∷ κ ∷ έ ∷ τ ∷ ι ∷ []) "John.5.14"
∷ word (ἁ ∷ μ ∷ ά ∷ ρ ∷ τ ∷ α ∷ ν ∷ ε ∷ []) "John.5.14"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.5.14"
∷ word (μ ∷ ὴ ∷ []) "John.5.14"
∷ word (χ ∷ ε ∷ ῖ ∷ ρ ∷ ό ∷ ν ∷ []) "John.5.14"
∷ word (σ ∷ ο ∷ ί ∷ []) "John.5.14"
∷ word (τ ∷ ι ∷ []) "John.5.14"
∷ word (γ ∷ έ ∷ ν ∷ η ∷ τ ∷ α ∷ ι ∷ []) "John.5.14"
∷ word (ἀ ∷ π ∷ ῆ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.5.15"
∷ word (ὁ ∷ []) "John.5.15"
∷ word (ἄ ∷ ν ∷ θ ∷ ρ ∷ ω ∷ π ∷ ο ∷ ς ∷ []) "John.5.15"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.5.15"
∷ word (ἀ ∷ ν ∷ ή ∷ γ ∷ γ ∷ ε ∷ ι ∷ ∙λ ∷ ε ∷ ν ∷ []) "John.5.15"
∷ word (τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.5.15"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ί ∷ ο ∷ ι ∷ ς ∷ []) "John.5.15"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.5.15"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.5.15"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.5.15"
∷ word (ὁ ∷ []) "John.5.15"
∷ word (π ∷ ο ∷ ι ∷ ή ∷ σ ∷ α ∷ ς ∷ []) "John.5.15"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.5.15"
∷ word (ὑ ∷ γ ∷ ι ∷ ῆ ∷ []) "John.5.15"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.5.16"
∷ word (δ ∷ ι ∷ ὰ ∷ []) "John.5.16"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.5.16"
∷ word (ἐ ∷ δ ∷ ί ∷ ω ∷ κ ∷ ο ∷ ν ∷ []) "John.5.16"
∷ word (ο ∷ ἱ ∷ []) "John.5.16"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ῖ ∷ ο ∷ ι ∷ []) "John.5.16"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.5.16"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ν ∷ []) "John.5.16"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.5.16"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.5.16"
∷ word (ἐ ∷ π ∷ ο ∷ ί ∷ ε ∷ ι ∷ []) "John.5.16"
∷ word (ἐ ∷ ν ∷ []) "John.5.16"
∷ word (σ ∷ α ∷ β ∷ β ∷ ά ∷ τ ∷ ῳ ∷ []) "John.5.16"
∷ word (ὁ ∷ []) "John.5.17"
∷ word (δ ∷ ὲ ∷ []) "John.5.17"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ ν ∷ α ∷ τ ∷ ο ∷ []) "John.5.17"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.5.17"
∷ word (Ὁ ∷ []) "John.5.17"
∷ word (π ∷ α ∷ τ ∷ ή ∷ ρ ∷ []) "John.5.17"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.5.17"
∷ word (ἕ ∷ ω ∷ ς ∷ []) "John.5.17"
∷ word (ἄ ∷ ρ ∷ τ ∷ ι ∷ []) "John.5.17"
∷ word (ἐ ∷ ρ ∷ γ ∷ ά ∷ ζ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.5.17"
∷ word (κ ∷ ἀ ∷ γ ∷ ὼ ∷ []) "John.5.17"
∷ word (ἐ ∷ ρ ∷ γ ∷ ά ∷ ζ ∷ ο ∷ μ ∷ α ∷ ι ∷ []) "John.5.17"
∷ word (δ ∷ ι ∷ ὰ ∷ []) "John.5.18"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.5.18"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.5.18"
∷ word (μ ∷ ᾶ ∷ ∙λ ∷ ∙λ ∷ ο ∷ ν ∷ []) "John.5.18"
∷ word (ἐ ∷ ζ ∷ ή ∷ τ ∷ ο ∷ υ ∷ ν ∷ []) "John.5.18"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.5.18"
∷ word (ο ∷ ἱ ∷ []) "John.5.18"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ῖ ∷ ο ∷ ι ∷ []) "John.5.18"
∷ word (ἀ ∷ π ∷ ο ∷ κ ∷ τ ∷ ε ∷ ῖ ∷ ν ∷ α ∷ ι ∷ []) "John.5.18"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.5.18"
∷ word (ο ∷ ὐ ∷ []) "John.5.18"
∷ word (μ ∷ ό ∷ ν ∷ ο ∷ ν ∷ []) "John.5.18"
∷ word (ἔ ∷ ∙λ ∷ υ ∷ ε ∷ []) "John.5.18"
∷ word (τ ∷ ὸ ∷ []) "John.5.18"
∷ word (σ ∷ ά ∷ β ∷ β ∷ α ∷ τ ∷ ο ∷ ν ∷ []) "John.5.18"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.5.18"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.5.18"
∷ word (π ∷ α ∷ τ ∷ έ ∷ ρ ∷ α ∷ []) "John.5.18"
∷ word (ἴ ∷ δ ∷ ι ∷ ο ∷ ν ∷ []) "John.5.18"
∷ word (ἔ ∷ ∙λ ∷ ε ∷ γ ∷ ε ∷ []) "John.5.18"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.5.18"
∷ word (θ ∷ ε ∷ ό ∷ ν ∷ []) "John.5.18"
∷ word (ἴ ∷ σ ∷ ο ∷ ν ∷ []) "John.5.18"
∷ word (ἑ ∷ α ∷ υ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.5.18"
∷ word (π ∷ ο ∷ ι ∷ ῶ ∷ ν ∷ []) "John.5.18"
∷ word (τ ∷ ῷ ∷ []) "John.5.18"
∷ word (θ ∷ ε ∷ ῷ ∷ []) "John.5.18"
∷ word (Ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ ν ∷ α ∷ τ ∷ ο ∷ []) "John.5.19"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.5.19"
∷ word (ὁ ∷ []) "John.5.19"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.5.19"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.5.19"
∷ word (ἔ ∷ ∙λ ∷ ε ∷ γ ∷ ε ∷ ν ∷ []) "John.5.19"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.5.19"
∷ word (Ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.5.19"
∷ word (ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.5.19"
∷ word (∙λ ∷ έ ∷ γ ∷ ω ∷ []) "John.5.19"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.5.19"
∷ word (ο ∷ ὐ ∷ []) "John.5.19"
∷ word (δ ∷ ύ ∷ ν ∷ α ∷ τ ∷ α ∷ ι ∷ []) "John.5.19"
∷ word (ὁ ∷ []) "John.5.19"
∷ word (υ ∷ ἱ ∷ ὸ ∷ ς ∷ []) "John.5.19"
∷ word (π ∷ ο ∷ ι ∷ ε ∷ ῖ ∷ ν ∷ []) "John.5.19"
∷ word (ἀ ∷ φ ∷ []) "John.5.19"
∷ word (ἑ ∷ α ∷ υ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.5.19"
∷ word (ο ∷ ὐ ∷ δ ∷ ὲ ∷ ν ∷ []) "John.5.19"
∷ word (ἐ ∷ ὰ ∷ ν ∷ []) "John.5.19"
∷ word (μ ∷ ή ∷ []) "John.5.19"
∷ word (τ ∷ ι ∷ []) "John.5.19"
∷ word (β ∷ ∙λ ∷ έ ∷ π ∷ ῃ ∷ []) "John.5.19"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.5.19"
∷ word (π ∷ α ∷ τ ∷ έ ∷ ρ ∷ α ∷ []) "John.5.19"
∷ word (π ∷ ο ∷ ι ∷ ο ∷ ῦ ∷ ν ∷ τ ∷ α ∷ []) "John.5.19"
∷ word (ἃ ∷ []) "John.5.19"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.5.19"
∷ word (ἂ ∷ ν ∷ []) "John.5.19"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ο ∷ ς ∷ []) "John.5.19"
∷ word (π ∷ ο ∷ ι ∷ ῇ ∷ []) "John.5.19"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.5.19"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.5.19"
∷ word (ὁ ∷ []) "John.5.19"
∷ word (υ ∷ ἱ ∷ ὸ ∷ ς ∷ []) "John.5.19"
∷ word (ὁ ∷ μ ∷ ο ∷ ί ∷ ω ∷ ς ∷ []) "John.5.19"
∷ word (π ∷ ο ∷ ι ∷ ε ∷ ῖ ∷ []) "John.5.19"
∷ word (ὁ ∷ []) "John.5.20"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.5.20"
∷ word (π ∷ α ∷ τ ∷ ὴ ∷ ρ ∷ []) "John.5.20"
∷ word (φ ∷ ι ∷ ∙λ ∷ ε ∷ ῖ ∷ []) "John.5.20"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.5.20"
∷ word (υ ∷ ἱ ∷ ὸ ∷ ν ∷ []) "John.5.20"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.5.20"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ α ∷ []) "John.5.20"
∷ word (δ ∷ ε ∷ ί ∷ κ ∷ ν ∷ υ ∷ σ ∷ ι ∷ ν ∷ []) "John.5.20"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.5.20"
∷ word (ἃ ∷ []) "John.5.20"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ς ∷ []) "John.5.20"
∷ word (π ∷ ο ∷ ι ∷ ε ∷ ῖ ∷ []) "John.5.20"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.5.20"
∷ word (μ ∷ ε ∷ ί ∷ ζ ∷ ο ∷ ν ∷ α ∷ []) "John.5.20"
∷ word (τ ∷ ο ∷ ύ ∷ τ ∷ ω ∷ ν ∷ []) "John.5.20"
∷ word (δ ∷ ε ∷ ί ∷ ξ ∷ ε ∷ ι ∷ []) "John.5.20"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.5.20"
∷ word (ἔ ∷ ρ ∷ γ ∷ α ∷ []) "John.5.20"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.5.20"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.5.20"
∷ word (θ ∷ α ∷ υ ∷ μ ∷ ά ∷ ζ ∷ η ∷ τ ∷ ε ∷ []) "John.5.20"
∷ word (ὥ ∷ σ ∷ π ∷ ε ∷ ρ ∷ []) "John.5.21"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.5.21"
∷ word (ὁ ∷ []) "John.5.21"
∷ word (π ∷ α ∷ τ ∷ ὴ ∷ ρ ∷ []) "John.5.21"
∷ word (ἐ ∷ γ ∷ ε ∷ ί ∷ ρ ∷ ε ∷ ι ∷ []) "John.5.21"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.5.21"
∷ word (ν ∷ ε ∷ κ ∷ ρ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.5.21"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.5.21"
∷ word (ζ ∷ ῳ ∷ ο ∷ π ∷ ο ∷ ι ∷ ε ∷ ῖ ∷ []) "John.5.21"
∷ word (ο ∷ ὕ ∷ τ ∷ ω ∷ ς ∷ []) "John.5.21"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.5.21"
∷ word (ὁ ∷ []) "John.5.21"
∷ word (υ ∷ ἱ ∷ ὸ ∷ ς ∷ []) "John.5.21"
∷ word (ο ∷ ὓ ∷ ς ∷ []) "John.5.21"
∷ word (θ ∷ έ ∷ ∙λ ∷ ε ∷ ι ∷ []) "John.5.21"
∷ word (ζ ∷ ῳ ∷ ο ∷ π ∷ ο ∷ ι ∷ ε ∷ ῖ ∷ []) "John.5.21"
∷ word (ο ∷ ὐ ∷ δ ∷ ὲ ∷ []) "John.5.22"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.5.22"
∷ word (ὁ ∷ []) "John.5.22"
∷ word (π ∷ α ∷ τ ∷ ὴ ∷ ρ ∷ []) "John.5.22"
∷ word (κ ∷ ρ ∷ ί ∷ ν ∷ ε ∷ ι ∷ []) "John.5.22"
∷ word (ο ∷ ὐ ∷ δ ∷ έ ∷ ν ∷ α ∷ []) "John.5.22"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.5.22"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.5.22"
∷ word (κ ∷ ρ ∷ ί ∷ σ ∷ ι ∷ ν ∷ []) "John.5.22"
∷ word (π ∷ ᾶ ∷ σ ∷ α ∷ ν ∷ []) "John.5.22"
∷ word (δ ∷ έ ∷ δ ∷ ω ∷ κ ∷ ε ∷ ν ∷ []) "John.5.22"
∷ word (τ ∷ ῷ ∷ []) "John.5.22"
∷ word (υ ∷ ἱ ∷ ῷ ∷ []) "John.5.22"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.5.23"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.5.23"
∷ word (τ ∷ ι ∷ μ ∷ ῶ ∷ σ ∷ ι ∷ []) "John.5.23"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.5.23"
∷ word (υ ∷ ἱ ∷ ὸ ∷ ν ∷ []) "John.5.23"
∷ word (κ ∷ α ∷ θ ∷ ὼ ∷ ς ∷ []) "John.5.23"
∷ word (τ ∷ ι ∷ μ ∷ ῶ ∷ σ ∷ ι ∷ []) "John.5.23"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.5.23"
∷ word (π ∷ α ∷ τ ∷ έ ∷ ρ ∷ α ∷ []) "John.5.23"
∷ word (ὁ ∷ []) "John.5.23"
∷ word (μ ∷ ὴ ∷ []) "John.5.23"
∷ word (τ ∷ ι ∷ μ ∷ ῶ ∷ ν ∷ []) "John.5.23"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.5.23"
∷ word (υ ∷ ἱ ∷ ὸ ∷ ν ∷ []) "John.5.23"
∷ word (ο ∷ ὐ ∷ []) "John.5.23"
∷ word (τ ∷ ι ∷ μ ∷ ᾷ ∷ []) "John.5.23"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.5.23"
∷ word (π ∷ α ∷ τ ∷ έ ∷ ρ ∷ α ∷ []) "John.5.23"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.5.23"
∷ word (π ∷ έ ∷ μ ∷ ψ ∷ α ∷ ν ∷ τ ∷ α ∷ []) "John.5.23"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.5.23"
∷ word (Ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.5.24"
∷ word (ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.5.24"
∷ word (∙λ ∷ έ ∷ γ ∷ ω ∷ []) "John.5.24"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.5.24"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.5.24"
∷ word (ὁ ∷ []) "John.5.24"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.5.24"
∷ word (∙λ ∷ ό ∷ γ ∷ ο ∷ ν ∷ []) "John.5.24"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.5.24"
∷ word (ἀ ∷ κ ∷ ο ∷ ύ ∷ ω ∷ ν ∷ []) "John.5.24"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.5.24"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ ω ∷ ν ∷ []) "John.5.24"
∷ word (τ ∷ ῷ ∷ []) "John.5.24"
∷ word (π ∷ έ ∷ μ ∷ ψ ∷ α ∷ ν ∷ τ ∷ ί ∷ []) "John.5.24"
∷ word (μ ∷ ε ∷ []) "John.5.24"
∷ word (ἔ ∷ χ ∷ ε ∷ ι ∷ []) "John.5.24"
∷ word (ζ ∷ ω ∷ ὴ ∷ ν ∷ []) "John.5.24"
∷ word (α ∷ ἰ ∷ ώ ∷ ν ∷ ι ∷ ο ∷ ν ∷ []) "John.5.24"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.5.24"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.5.24"
∷ word (κ ∷ ρ ∷ ί ∷ σ ∷ ι ∷ ν ∷ []) "John.5.24"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.5.24"
∷ word (ἔ ∷ ρ ∷ χ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.5.24"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.5.24"
∷ word (μ ∷ ε ∷ τ ∷ α ∷ β ∷ έ ∷ β ∷ η ∷ κ ∷ ε ∷ ν ∷ []) "John.5.24"
∷ word (ἐ ∷ κ ∷ []) "John.5.24"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.5.24"
∷ word (θ ∷ α ∷ ν ∷ ά ∷ τ ∷ ο ∷ υ ∷ []) "John.5.24"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.5.24"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.5.24"
∷ word (ζ ∷ ω ∷ ή ∷ ν ∷ []) "John.5.24"
∷ word (Ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.5.25"
∷ word (ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.5.25"
∷ word (∙λ ∷ έ ∷ γ ∷ ω ∷ []) "John.5.25"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.5.25"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.5.25"
∷ word (ἔ ∷ ρ ∷ χ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.5.25"
∷ word (ὥ ∷ ρ ∷ α ∷ []) "John.5.25"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.5.25"
∷ word (ν ∷ ῦ ∷ ν ∷ []) "John.5.25"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.5.25"
∷ word (ὅ ∷ τ ∷ ε ∷ []) "John.5.25"
∷ word (ο ∷ ἱ ∷ []) "John.5.25"
∷ word (ν ∷ ε ∷ κ ∷ ρ ∷ ο ∷ ὶ ∷ []) "John.5.25"
∷ word (ἀ ∷ κ ∷ ο ∷ ύ ∷ σ ∷ ο ∷ υ ∷ σ ∷ ι ∷ ν ∷ []) "John.5.25"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.5.25"
∷ word (φ ∷ ω ∷ ν ∷ ῆ ∷ ς ∷ []) "John.5.25"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.5.25"
∷ word (υ ∷ ἱ ∷ ο ∷ ῦ ∷ []) "John.5.25"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.5.25"
∷ word (θ ∷ ε ∷ ο ∷ ῦ ∷ []) "John.5.25"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.5.25"
∷ word (ο ∷ ἱ ∷ []) "John.5.25"
∷ word (ἀ ∷ κ ∷ ο ∷ ύ ∷ σ ∷ α ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.5.25"
∷ word (ζ ∷ ή ∷ σ ∷ ο ∷ υ ∷ σ ∷ ι ∷ ν ∷ []) "John.5.25"
∷ word (ὥ ∷ σ ∷ π ∷ ε ∷ ρ ∷ []) "John.5.26"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.5.26"
∷ word (ὁ ∷ []) "John.5.26"
∷ word (π ∷ α ∷ τ ∷ ὴ ∷ ρ ∷ []) "John.5.26"
∷ word (ἔ ∷ χ ∷ ε ∷ ι ∷ []) "John.5.26"
∷ word (ζ ∷ ω ∷ ὴ ∷ ν ∷ []) "John.5.26"
∷ word (ἐ ∷ ν ∷ []) "John.5.26"
∷ word (ἑ ∷ α ∷ υ ∷ τ ∷ ῷ ∷ []) "John.5.26"
∷ word (ο ∷ ὕ ∷ τ ∷ ω ∷ ς ∷ []) "John.5.26"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.5.26"
∷ word (τ ∷ ῷ ∷ []) "John.5.26"
∷ word (υ ∷ ἱ ∷ ῷ ∷ []) "John.5.26"
∷ word (ἔ ∷ δ ∷ ω ∷ κ ∷ ε ∷ ν ∷ []) "John.5.26"
∷ word (ζ ∷ ω ∷ ὴ ∷ ν ∷ []) "John.5.26"
∷ word (ἔ ∷ χ ∷ ε ∷ ι ∷ ν ∷ []) "John.5.26"
∷ word (ἐ ∷ ν ∷ []) "John.5.26"
∷ word (ἑ ∷ α ∷ υ ∷ τ ∷ ῷ ∷ []) "John.5.26"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.5.27"
∷ word (ἐ ∷ ξ ∷ ο ∷ υ ∷ σ ∷ ί ∷ α ∷ ν ∷ []) "John.5.27"
∷ word (ἔ ∷ δ ∷ ω ∷ κ ∷ ε ∷ ν ∷ []) "John.5.27"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.5.27"
∷ word (κ ∷ ρ ∷ ί ∷ σ ∷ ι ∷ ν ∷ []) "John.5.27"
∷ word (π ∷ ο ∷ ι ∷ ε ∷ ῖ ∷ ν ∷ []) "John.5.27"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.5.27"
∷ word (υ ∷ ἱ ∷ ὸ ∷ ς ∷ []) "John.5.27"
∷ word (ἀ ∷ ν ∷ θ ∷ ρ ∷ ώ ∷ π ∷ ο ∷ υ ∷ []) "John.5.27"
∷ word (ἐ ∷ σ ∷ τ ∷ ί ∷ ν ∷ []) "John.5.27"
∷ word (μ ∷ ὴ ∷ []) "John.5.28"
∷ word (θ ∷ α ∷ υ ∷ μ ∷ ά ∷ ζ ∷ ε ∷ τ ∷ ε ∷ []) "John.5.28"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.5.28"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.5.28"
∷ word (ἔ ∷ ρ ∷ χ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.5.28"
∷ word (ὥ ∷ ρ ∷ α ∷ []) "John.5.28"
∷ word (ἐ ∷ ν ∷ []) "John.5.28"
∷ word (ᾗ ∷ []) "John.5.28"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.5.28"
∷ word (ο ∷ ἱ ∷ []) "John.5.28"
∷ word (ἐ ∷ ν ∷ []) "John.5.28"
∷ word (τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.5.28"
∷ word (μ ∷ ν ∷ η ∷ μ ∷ ε ∷ ί ∷ ο ∷ ι ∷ ς ∷ []) "John.5.28"
∷ word (ἀ ∷ κ ∷ ο ∷ ύ ∷ σ ∷ ο ∷ υ ∷ σ ∷ ι ∷ ν ∷ []) "John.5.28"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.5.28"
∷ word (φ ∷ ω ∷ ν ∷ ῆ ∷ ς ∷ []) "John.5.28"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.5.28"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.5.29"
∷ word (ἐ ∷ κ ∷ π ∷ ο ∷ ρ ∷ ε ∷ ύ ∷ σ ∷ ο ∷ ν ∷ τ ∷ α ∷ ι ∷ []) "John.5.29"
∷ word (ο ∷ ἱ ∷ []) "John.5.29"
∷ word (τ ∷ ὰ ∷ []) "John.5.29"
∷ word (ἀ ∷ γ ∷ α ∷ θ ∷ ὰ ∷ []) "John.5.29"
∷ word (π ∷ ο ∷ ι ∷ ή ∷ σ ∷ α ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.5.29"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.5.29"
∷ word (ἀ ∷ ν ∷ ά ∷ σ ∷ τ ∷ α ∷ σ ∷ ι ∷ ν ∷ []) "John.5.29"
∷ word (ζ ∷ ω ∷ ῆ ∷ ς ∷ []) "John.5.29"
∷ word (ο ∷ ἱ ∷ []) "John.5.29"
∷ word (δ ∷ ὲ ∷ []) "John.5.29"
∷ word (τ ∷ ὰ ∷ []) "John.5.29"
∷ word (φ ∷ α ∷ ῦ ∷ ∙λ ∷ α ∷ []) "John.5.29"
∷ word (π ∷ ρ ∷ ά ∷ ξ ∷ α ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.5.29"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.5.29"
∷ word (ἀ ∷ ν ∷ ά ∷ σ ∷ τ ∷ α ∷ σ ∷ ι ∷ ν ∷ []) "John.5.29"
∷ word (κ ∷ ρ ∷ ί ∷ σ ∷ ε ∷ ω ∷ ς ∷ []) "John.5.29"
∷ word (Ο ∷ ὐ ∷ []) "John.5.30"
∷ word (δ ∷ ύ ∷ ν ∷ α ∷ μ ∷ α ∷ ι ∷ []) "John.5.30"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.5.30"
∷ word (π ∷ ο ∷ ι ∷ ε ∷ ῖ ∷ ν ∷ []) "John.5.30"
∷ word (ἀ ∷ π ∷ []) "John.5.30"
∷ word (ἐ ∷ μ ∷ α ∷ υ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.5.30"
∷ word (ο ∷ ὐ ∷ δ ∷ έ ∷ ν ∷ []) "John.5.30"
∷ word (κ ∷ α ∷ θ ∷ ὼ ∷ ς ∷ []) "John.5.30"
∷ word (ἀ ∷ κ ∷ ο ∷ ύ ∷ ω ∷ []) "John.5.30"
∷ word (κ ∷ ρ ∷ ί ∷ ν ∷ ω ∷ []) "John.5.30"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.5.30"
∷ word (ἡ ∷ []) "John.5.30"
∷ word (κ ∷ ρ ∷ ί ∷ σ ∷ ι ∷ ς ∷ []) "John.5.30"
∷ word (ἡ ∷ []) "John.5.30"
∷ word (ἐ ∷ μ ∷ ὴ ∷ []) "John.5.30"
∷ word (δ ∷ ι ∷ κ ∷ α ∷ ί ∷ α ∷ []) "John.5.30"
∷ word (ἐ ∷ σ ∷ τ ∷ ί ∷ ν ∷ []) "John.5.30"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.5.30"
∷ word (ο ∷ ὐ ∷ []) "John.5.30"
∷ word (ζ ∷ η ∷ τ ∷ ῶ ∷ []) "John.5.30"
∷ word (τ ∷ ὸ ∷ []) "John.5.30"
∷ word (θ ∷ έ ∷ ∙λ ∷ η ∷ μ ∷ α ∷ []) "John.5.30"
∷ word (τ ∷ ὸ ∷ []) "John.5.30"
∷ word (ἐ ∷ μ ∷ ὸ ∷ ν ∷ []) "John.5.30"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.5.30"
∷ word (τ ∷ ὸ ∷ []) "John.5.30"
∷ word (θ ∷ έ ∷ ∙λ ∷ η ∷ μ ∷ α ∷ []) "John.5.30"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.5.30"
∷ word (π ∷ έ ∷ μ ∷ ψ ∷ α ∷ ν ∷ τ ∷ ό ∷ ς ∷ []) "John.5.30"
∷ word (μ ∷ ε ∷ []) "John.5.30"
∷ word (Ἐ ∷ ὰ ∷ ν ∷ []) "John.5.31"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.5.31"
∷ word (μ ∷ α ∷ ρ ∷ τ ∷ υ ∷ ρ ∷ ῶ ∷ []) "John.5.31"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.5.31"
∷ word (ἐ ∷ μ ∷ α ∷ υ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.5.31"
∷ word (ἡ ∷ []) "John.5.31"
∷ word (μ ∷ α ∷ ρ ∷ τ ∷ υ ∷ ρ ∷ ί ∷ α ∷ []) "John.5.31"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.5.31"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.5.31"
∷ word (ἔ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.5.31"
∷ word (ἀ ∷ ∙λ ∷ η ∷ θ ∷ ή ∷ ς ∷ []) "John.5.31"
∷ word (ἄ ∷ ∙λ ∷ ∙λ ∷ ο ∷ ς ∷ []) "John.5.32"
∷ word (ἐ ∷ σ ∷ τ ∷ ὶ ∷ ν ∷ []) "John.5.32"
∷ word (ὁ ∷ []) "John.5.32"
∷ word (μ ∷ α ∷ ρ ∷ τ ∷ υ ∷ ρ ∷ ῶ ∷ ν ∷ []) "John.5.32"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.5.32"
∷ word (ἐ ∷ μ ∷ ο ∷ ῦ ∷ []) "John.5.32"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.5.32"
∷ word (ο ∷ ἶ ∷ δ ∷ α ∷ []) "John.5.32"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.5.32"
∷ word (ἀ ∷ ∙λ ∷ η ∷ θ ∷ ή ∷ ς ∷ []) "John.5.32"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.5.32"
∷ word (ἡ ∷ []) "John.5.32"
∷ word (μ ∷ α ∷ ρ ∷ τ ∷ υ ∷ ρ ∷ ί ∷ α ∷ []) "John.5.32"
∷ word (ἣ ∷ ν ∷ []) "John.5.32"
∷ word (μ ∷ α ∷ ρ ∷ τ ∷ υ ∷ ρ ∷ ε ∷ ῖ ∷ []) "John.5.32"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.5.32"
∷ word (ἐ ∷ μ ∷ ο ∷ ῦ ∷ []) "John.5.32"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.5.33"
∷ word (ἀ ∷ π ∷ ε ∷ σ ∷ τ ∷ ά ∷ ∙λ ∷ κ ∷ α ∷ τ ∷ ε ∷ []) "John.5.33"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.5.33"
∷ word (Ἰ ∷ ω ∷ ά ∷ ν ∷ ν ∷ η ∷ ν ∷ []) "John.5.33"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.5.33"
∷ word (μ ∷ ε ∷ μ ∷ α ∷ ρ ∷ τ ∷ ύ ∷ ρ ∷ η ∷ κ ∷ ε ∷ []) "John.5.33"
∷ word (τ ∷ ῇ ∷ []) "John.5.33"
∷ word (ἀ ∷ ∙λ ∷ η ∷ θ ∷ ε ∷ ί ∷ ᾳ ∷ []) "John.5.33"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.5.34"
∷ word (δ ∷ ὲ ∷ []) "John.5.34"
∷ word (ο ∷ ὐ ∷ []) "John.5.34"
∷ word (π ∷ α ∷ ρ ∷ ὰ ∷ []) "John.5.34"
∷ word (ἀ ∷ ν ∷ θ ∷ ρ ∷ ώ ∷ π ∷ ο ∷ υ ∷ []) "John.5.34"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.5.34"
∷ word (μ ∷ α ∷ ρ ∷ τ ∷ υ ∷ ρ ∷ ί ∷ α ∷ ν ∷ []) "John.5.34"
∷ word (∙λ ∷ α ∷ μ ∷ β ∷ ά ∷ ν ∷ ω ∷ []) "John.5.34"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.5.34"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.5.34"
∷ word (∙λ ∷ έ ∷ γ ∷ ω ∷ []) "John.5.34"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.5.34"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.5.34"
∷ word (σ ∷ ω ∷ θ ∷ ῆ ∷ τ ∷ ε ∷ []) "John.5.34"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ο ∷ ς ∷ []) "John.5.35"
∷ word (ἦ ∷ ν ∷ []) "John.5.35"
∷ word (ὁ ∷ []) "John.5.35"
∷ word (∙λ ∷ ύ ∷ χ ∷ ν ∷ ο ∷ ς ∷ []) "John.5.35"
∷ word (ὁ ∷ []) "John.5.35"
∷ word (κ ∷ α ∷ ι ∷ ό ∷ μ ∷ ε ∷ ν ∷ ο ∷ ς ∷ []) "John.5.35"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.5.35"
∷ word (φ ∷ α ∷ ί ∷ ν ∷ ω ∷ ν ∷ []) "John.5.35"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.5.35"
∷ word (δ ∷ ὲ ∷ []) "John.5.35"
∷ word (ἠ ∷ θ ∷ ε ∷ ∙λ ∷ ή ∷ σ ∷ α ∷ τ ∷ ε ∷ []) "John.5.35"
∷ word (ἀ ∷ γ ∷ α ∷ ∙λ ∷ ∙λ ∷ ι ∷ α ∷ θ ∷ ῆ ∷ ν ∷ α ∷ ι ∷ []) "John.5.35"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.5.35"
∷ word (ὥ ∷ ρ ∷ α ∷ ν ∷ []) "John.5.35"
∷ word (ἐ ∷ ν ∷ []) "John.5.35"
∷ word (τ ∷ ῷ ∷ []) "John.5.35"
∷ word (φ ∷ ω ∷ τ ∷ ὶ ∷ []) "John.5.35"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.5.35"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.5.36"
∷ word (δ ∷ ὲ ∷ []) "John.5.36"
∷ word (ἔ ∷ χ ∷ ω ∷ []) "John.5.36"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.5.36"
∷ word (μ ∷ α ∷ ρ ∷ τ ∷ υ ∷ ρ ∷ ί ∷ α ∷ ν ∷ []) "John.5.36"
∷ word (μ ∷ ε ∷ ί ∷ ζ ∷ ω ∷ []) "John.5.36"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.5.36"
∷ word (Ἰ ∷ ω ∷ ά ∷ ν ∷ ν ∷ ο ∷ υ ∷ []) "John.5.36"
∷ word (τ ∷ ὰ ∷ []) "John.5.36"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.5.36"
∷ word (ἔ ∷ ρ ∷ γ ∷ α ∷ []) "John.5.36"
∷ word (ἃ ∷ []) "John.5.36"
∷ word (δ ∷ έ ∷ δ ∷ ω ∷ κ ∷ έ ∷ ν ∷ []) "John.5.36"
∷ word (μ ∷ ο ∷ ι ∷ []) "John.5.36"
∷ word (ὁ ∷ []) "John.5.36"
∷ word (π ∷ α ∷ τ ∷ ὴ ∷ ρ ∷ []) "John.5.36"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.5.36"
∷ word (τ ∷ ε ∷ ∙λ ∷ ε ∷ ι ∷ ώ ∷ σ ∷ ω ∷ []) "John.5.36"
∷ word (α ∷ ὐ ∷ τ ∷ ά ∷ []) "John.5.36"
∷ word (α ∷ ὐ ∷ τ ∷ ὰ ∷ []) "John.5.36"
∷ word (τ ∷ ὰ ∷ []) "John.5.36"
∷ word (ἔ ∷ ρ ∷ γ ∷ α ∷ []) "John.5.36"
∷ word (ἃ ∷ []) "John.5.36"
∷ word (π ∷ ο ∷ ι ∷ ῶ ∷ []) "John.5.36"
∷ word (μ ∷ α ∷ ρ ∷ τ ∷ υ ∷ ρ ∷ ε ∷ ῖ ∷ []) "John.5.36"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.5.36"
∷ word (ἐ ∷ μ ∷ ο ∷ ῦ ∷ []) "John.5.36"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.5.36"
∷ word (ὁ ∷ []) "John.5.36"
∷ word (π ∷ α ∷ τ ∷ ή ∷ ρ ∷ []) "John.5.36"
∷ word (μ ∷ ε ∷ []) "John.5.36"
∷ word (ἀ ∷ π ∷ έ ∷ σ ∷ τ ∷ α ∷ ∙λ ∷ κ ∷ ε ∷ ν ∷ []) "John.5.36"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.5.37"
∷ word (ὁ ∷ []) "John.5.37"
∷ word (π ∷ έ ∷ μ ∷ ψ ∷ α ∷ ς ∷ []) "John.5.37"
∷ word (μ ∷ ε ∷ []) "John.5.37"
∷ word (π ∷ α ∷ τ ∷ ὴ ∷ ρ ∷ []) "John.5.37"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ο ∷ ς ∷ []) "John.5.37"
∷ word (μ ∷ ε ∷ μ ∷ α ∷ ρ ∷ τ ∷ ύ ∷ ρ ∷ η ∷ κ ∷ ε ∷ ν ∷ []) "John.5.37"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.5.37"
∷ word (ἐ ∷ μ ∷ ο ∷ ῦ ∷ []) "John.5.37"
∷ word (ο ∷ ὔ ∷ τ ∷ ε ∷ []) "John.5.37"
∷ word (φ ∷ ω ∷ ν ∷ ὴ ∷ ν ∷ []) "John.5.37"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.5.37"
∷ word (π ∷ ώ ∷ π ∷ ο ∷ τ ∷ ε ∷ []) "John.5.37"
∷ word (ἀ ∷ κ ∷ η ∷ κ ∷ ό ∷ α ∷ τ ∷ ε ∷ []) "John.5.37"
∷ word (ο ∷ ὔ ∷ τ ∷ ε ∷ []) "John.5.37"
∷ word (ε ∷ ἶ ∷ δ ∷ ο ∷ ς ∷ []) "John.5.37"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.5.37"
∷ word (ἑ ∷ ω ∷ ρ ∷ ά ∷ κ ∷ α ∷ τ ∷ ε ∷ []) "John.5.37"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.5.38"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.5.38"
∷ word (∙λ ∷ ό ∷ γ ∷ ο ∷ ν ∷ []) "John.5.38"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.5.38"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.5.38"
∷ word (ἔ ∷ χ ∷ ε ∷ τ ∷ ε ∷ []) "John.5.38"
∷ word (ἐ ∷ ν ∷ []) "John.5.38"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.5.38"
∷ word (μ ∷ έ ∷ ν ∷ ο ∷ ν ∷ τ ∷ α ∷ []) "John.5.38"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.5.38"
∷ word (ὃ ∷ ν ∷ []) "John.5.38"
∷ word (ἀ ∷ π ∷ έ ∷ σ ∷ τ ∷ ε ∷ ι ∷ ∙λ ∷ ε ∷ ν ∷ []) "John.5.38"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ο ∷ ς ∷ []) "John.5.38"
∷ word (τ ∷ ο ∷ ύ ∷ τ ∷ ῳ ∷ []) "John.5.38"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.5.38"
∷ word (ο ∷ ὐ ∷ []) "John.5.38"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ ε ∷ τ ∷ ε ∷ []) "John.5.38"
∷ word (Ἐ ∷ ρ ∷ α ∷ υ ∷ ν ∷ ᾶ ∷ τ ∷ ε ∷ []) "John.5.39"
∷ word (τ ∷ ὰ ∷ ς ∷ []) "John.5.39"
∷ word (γ ∷ ρ ∷ α ∷ φ ∷ ά ∷ ς ∷ []) "John.5.39"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.5.39"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.5.39"
∷ word (δ ∷ ο ∷ κ ∷ ε ∷ ῖ ∷ τ ∷ ε ∷ []) "John.5.39"
∷ word (ἐ ∷ ν ∷ []) "John.5.39"
∷ word (α ∷ ὐ ∷ τ ∷ α ∷ ῖ ∷ ς ∷ []) "John.5.39"
∷ word (ζ ∷ ω ∷ ὴ ∷ ν ∷ []) "John.5.39"
∷ word (α ∷ ἰ ∷ ώ ∷ ν ∷ ι ∷ ο ∷ ν ∷ []) "John.5.39"
∷ word (ἔ ∷ χ ∷ ε ∷ ι ∷ ν ∷ []) "John.5.39"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.5.39"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ α ∷ ί ∷ []) "John.5.39"
∷ word (ε ∷ ἰ ∷ σ ∷ ι ∷ ν ∷ []) "John.5.39"
∷ word (α ∷ ἱ ∷ []) "John.5.39"
∷ word (μ ∷ α ∷ ρ ∷ τ ∷ υ ∷ ρ ∷ ο ∷ ῦ ∷ σ ∷ α ∷ ι ∷ []) "John.5.39"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.5.39"
∷ word (ἐ ∷ μ ∷ ο ∷ ῦ ∷ []) "John.5.39"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.5.40"
∷ word (ο ∷ ὐ ∷ []) "John.5.40"
∷ word (θ ∷ έ ∷ ∙λ ∷ ε ∷ τ ∷ ε ∷ []) "John.5.40"
∷ word (ἐ ∷ ∙λ ∷ θ ∷ ε ∷ ῖ ∷ ν ∷ []) "John.5.40"
∷ word (π ∷ ρ ∷ ό ∷ ς ∷ []) "John.5.40"
∷ word (μ ∷ ε ∷ []) "John.5.40"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.5.40"
∷ word (ζ ∷ ω ∷ ὴ ∷ ν ∷ []) "John.5.40"
∷ word (ἔ ∷ χ ∷ η ∷ τ ∷ ε ∷ []) "John.5.40"
∷ word (δ ∷ ό ∷ ξ ∷ α ∷ ν ∷ []) "John.5.41"
∷ word (π ∷ α ∷ ρ ∷ ὰ ∷ []) "John.5.41"
∷ word (ἀ ∷ ν ∷ θ ∷ ρ ∷ ώ ∷ π ∷ ω ∷ ν ∷ []) "John.5.41"
∷ word (ο ∷ ὐ ∷ []) "John.5.41"
∷ word (∙λ ∷ α ∷ μ ∷ β ∷ ά ∷ ν ∷ ω ∷ []) "John.5.41"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.5.42"
∷ word (ἔ ∷ γ ∷ ν ∷ ω ∷ κ ∷ α ∷ []) "John.5.42"
∷ word (ὑ ∷ μ ∷ ᾶ ∷ ς ∷ []) "John.5.42"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.5.42"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.5.42"
∷ word (ἀ ∷ γ ∷ ά ∷ π ∷ η ∷ ν ∷ []) "John.5.42"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.5.42"
∷ word (θ ∷ ε ∷ ο ∷ ῦ ∷ []) "John.5.42"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.5.42"
∷ word (ἔ ∷ χ ∷ ε ∷ τ ∷ ε ∷ []) "John.5.42"
∷ word (ἐ ∷ ν ∷ []) "John.5.42"
∷ word (ἑ ∷ α ∷ υ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.5.42"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.5.43"
∷ word (ἐ ∷ ∙λ ∷ ή ∷ ∙λ ∷ υ ∷ θ ∷ α ∷ []) "John.5.43"
∷ word (ἐ ∷ ν ∷ []) "John.5.43"
∷ word (τ ∷ ῷ ∷ []) "John.5.43"
∷ word (ὀ ∷ ν ∷ ό ∷ μ ∷ α ∷ τ ∷ ι ∷ []) "John.5.43"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.5.43"
∷ word (π ∷ α ∷ τ ∷ ρ ∷ ό ∷ ς ∷ []) "John.5.43"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.5.43"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.5.43"
∷ word (ο ∷ ὐ ∷ []) "John.5.43"
∷ word (∙λ ∷ α ∷ μ ∷ β ∷ ά ∷ ν ∷ ε ∷ τ ∷ έ ∷ []) "John.5.43"
∷ word (μ ∷ ε ∷ []) "John.5.43"
∷ word (ἐ ∷ ὰ ∷ ν ∷ []) "John.5.43"
∷ word (ἄ ∷ ∙λ ∷ ∙λ ∷ ο ∷ ς ∷ []) "John.5.43"
∷ word (ἔ ∷ ∙λ ∷ θ ∷ ῃ ∷ []) "John.5.43"
∷ word (ἐ ∷ ν ∷ []) "John.5.43"
∷ word (τ ∷ ῷ ∷ []) "John.5.43"
∷ word (ὀ ∷ ν ∷ ό ∷ μ ∷ α ∷ τ ∷ ι ∷ []) "John.5.43"
∷ word (τ ∷ ῷ ∷ []) "John.5.43"
∷ word (ἰ ∷ δ ∷ ί ∷ ῳ ∷ []) "John.5.43"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ο ∷ ν ∷ []) "John.5.43"
∷ word (∙λ ∷ ή ∷ μ ∷ ψ ∷ ε ∷ σ ∷ θ ∷ ε ∷ []) "John.5.43"
∷ word (π ∷ ῶ ∷ ς ∷ []) "John.5.44"
∷ word (δ ∷ ύ ∷ ν ∷ α ∷ σ ∷ θ ∷ ε ∷ []) "John.5.44"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.5.44"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ῦ ∷ σ ∷ α ∷ ι ∷ []) "John.5.44"
∷ word (δ ∷ ό ∷ ξ ∷ α ∷ ν ∷ []) "John.5.44"
∷ word (π ∷ α ∷ ρ ∷ []) "John.5.44"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ή ∷ ∙λ ∷ ω ∷ ν ∷ []) "John.5.44"
∷ word (∙λ ∷ α ∷ μ ∷ β ∷ ά ∷ ν ∷ ο ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.5.44"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.5.44"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.5.44"
∷ word (δ ∷ ό ∷ ξ ∷ α ∷ ν ∷ []) "John.5.44"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.5.44"
∷ word (π ∷ α ∷ ρ ∷ ὰ ∷ []) "John.5.44"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.5.44"
∷ word (μ ∷ ό ∷ ν ∷ ο ∷ υ ∷ []) "John.5.44"
∷ word (θ ∷ ε ∷ ο ∷ ῦ ∷ []) "John.5.44"
∷ word (ο ∷ ὐ ∷ []) "John.5.44"
∷ word (ζ ∷ η ∷ τ ∷ ε ∷ ῖ ∷ τ ∷ ε ∷ []) "John.5.44"
∷ word (μ ∷ ὴ ∷ []) "John.5.45"
∷ word (δ ∷ ο ∷ κ ∷ ε ∷ ῖ ∷ τ ∷ ε ∷ []) "John.5.45"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.5.45"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.5.45"
∷ word (κ ∷ α ∷ τ ∷ η ∷ γ ∷ ο ∷ ρ ∷ ή ∷ σ ∷ ω ∷ []) "John.5.45"
∷ word (ὑ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.5.45"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.5.45"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.5.45"
∷ word (π ∷ α ∷ τ ∷ έ ∷ ρ ∷ α ∷ []) "John.5.45"
∷ word (ἔ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.5.45"
∷ word (ὁ ∷ []) "John.5.45"
∷ word (κ ∷ α ∷ τ ∷ η ∷ γ ∷ ο ∷ ρ ∷ ῶ ∷ ν ∷ []) "John.5.45"
∷ word (ὑ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.5.45"
∷ word (Μ ∷ ω ∷ ϋ ∷ σ ∷ ῆ ∷ ς ∷ []) "John.5.45"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.5.45"
∷ word (ὃ ∷ ν ∷ []) "John.5.45"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.5.45"
∷ word (ἠ ∷ ∙λ ∷ π ∷ ί ∷ κ ∷ α ∷ τ ∷ ε ∷ []) "John.5.45"
∷ word (ε ∷ ἰ ∷ []) "John.5.46"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.5.46"
∷ word (ἐ ∷ π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ ε ∷ τ ∷ ε ∷ []) "John.5.46"
∷ word (Μ ∷ ω ∷ ϋ ∷ σ ∷ ε ∷ ῖ ∷ []) "John.5.46"
∷ word (ἐ ∷ π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ ε ∷ τ ∷ ε ∷ []) "John.5.46"
∷ word (ἂ ∷ ν ∷ []) "John.5.46"
∷ word (ἐ ∷ μ ∷ ο ∷ ί ∷ []) "John.5.46"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.5.46"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.5.46"
∷ word (ἐ ∷ μ ∷ ο ∷ ῦ ∷ []) "John.5.46"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ο ∷ ς ∷ []) "John.5.46"
∷ word (ἔ ∷ γ ∷ ρ ∷ α ∷ ψ ∷ ε ∷ ν ∷ []) "John.5.46"
∷ word (ε ∷ ἰ ∷ []) "John.5.47"
∷ word (δ ∷ ὲ ∷ []) "John.5.47"
∷ word (τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.5.47"
∷ word (ἐ ∷ κ ∷ ε ∷ ί ∷ ν ∷ ο ∷ υ ∷ []) "John.5.47"
∷ word (γ ∷ ρ ∷ ά ∷ μ ∷ μ ∷ α ∷ σ ∷ ι ∷ ν ∷ []) "John.5.47"
∷ word (ο ∷ ὐ ∷ []) "John.5.47"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ ε ∷ τ ∷ ε ∷ []) "John.5.47"
∷ word (π ∷ ῶ ∷ ς ∷ []) "John.5.47"
∷ word (τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.5.47"
∷ word (ἐ ∷ μ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.5.47"
∷ word (ῥ ∷ ή ∷ μ ∷ α ∷ σ ∷ ι ∷ ν ∷ []) "John.5.47"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ σ ∷ ε ∷ τ ∷ ε ∷ []) "John.5.47"
∷ word (Μ ∷ ε ∷ τ ∷ ὰ ∷ []) "John.6.1"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.6.1"
∷ word (ἀ ∷ π ∷ ῆ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.6.1"
∷ word (ὁ ∷ []) "John.6.1"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.6.1"
∷ word (π ∷ έ ∷ ρ ∷ α ∷ ν ∷ []) "John.6.1"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.6.1"
∷ word (θ ∷ α ∷ ∙λ ∷ ά ∷ σ ∷ σ ∷ η ∷ ς ∷ []) "John.6.1"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.6.1"
∷ word (Γ ∷ α ∷ ∙λ ∷ ι ∷ ∙λ ∷ α ∷ ί ∷ α ∷ ς ∷ []) "John.6.1"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.6.1"
∷ word (Τ ∷ ι ∷ β ∷ ε ∷ ρ ∷ ι ∷ ά ∷ δ ∷ ο ∷ ς ∷ []) "John.6.1"
∷ word (ἠ ∷ κ ∷ ο ∷ ∙λ ∷ ο ∷ ύ ∷ θ ∷ ε ∷ ι ∷ []) "John.6.2"
∷ word (δ ∷ ὲ ∷ []) "John.6.2"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.6.2"
∷ word (ὄ ∷ χ ∷ ∙λ ∷ ο ∷ ς ∷ []) "John.6.2"
∷ word (π ∷ ο ∷ ∙λ ∷ ύ ∷ ς ∷ []) "John.6.2"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.6.2"
∷ word (ἐ ∷ θ ∷ ε ∷ ώ ∷ ρ ∷ ο ∷ υ ∷ ν ∷ []) "John.6.2"
∷ word (τ ∷ ὰ ∷ []) "John.6.2"
∷ word (σ ∷ η ∷ μ ∷ ε ∷ ῖ ∷ α ∷ []) "John.6.2"
∷ word (ἃ ∷ []) "John.6.2"
∷ word (ἐ ∷ π ∷ ο ∷ ί ∷ ε ∷ ι ∷ []) "John.6.2"
∷ word (ἐ ∷ π ∷ ὶ ∷ []) "John.6.2"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.6.2"
∷ word (ἀ ∷ σ ∷ θ ∷ ε ∷ ν ∷ ο ∷ ύ ∷ ν ∷ τ ∷ ω ∷ ν ∷ []) "John.6.2"
∷ word (ἀ ∷ ν ∷ ῆ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.6.3"
∷ word (δ ∷ ὲ ∷ []) "John.6.3"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.6.3"
∷ word (τ ∷ ὸ ∷ []) "John.6.3"
∷ word (ὄ ∷ ρ ∷ ο ∷ ς ∷ []) "John.6.3"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.6.3"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.6.3"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ []) "John.6.3"
∷ word (ἐ ∷ κ ∷ ά ∷ θ ∷ η ∷ τ ∷ ο ∷ []) "John.6.3"
∷ word (μ ∷ ε ∷ τ ∷ ὰ ∷ []) "John.6.3"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.6.3"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ ῶ ∷ ν ∷ []) "John.6.3"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.6.3"
∷ word (ἦ ∷ ν ∷ []) "John.6.4"
∷ word (δ ∷ ὲ ∷ []) "John.6.4"
∷ word (ἐ ∷ γ ∷ γ ∷ ὺ ∷ ς ∷ []) "John.6.4"
∷ word (τ ∷ ὸ ∷ []) "John.6.4"
∷ word (π ∷ ά ∷ σ ∷ χ ∷ α ∷ []) "John.6.4"
∷ word (ἡ ∷ []) "John.6.4"
∷ word (ἑ ∷ ο ∷ ρ ∷ τ ∷ ὴ ∷ []) "John.6.4"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.6.4"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ί ∷ ω ∷ ν ∷ []) "John.6.4"
∷ word (ἐ ∷ π ∷ ά ∷ ρ ∷ α ∷ ς ∷ []) "John.6.5"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.6.5"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.6.5"
∷ word (ὀ ∷ φ ∷ θ ∷ α ∷ ∙λ ∷ μ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.6.5"
∷ word (ὁ ∷ []) "John.6.5"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.6.5"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.6.5"
∷ word (θ ∷ ε ∷ α ∷ σ ∷ ά ∷ μ ∷ ε ∷ ν ∷ ο ∷ ς ∷ []) "John.6.5"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.6.5"
∷ word (π ∷ ο ∷ ∙λ ∷ ὺ ∷ ς ∷ []) "John.6.5"
∷ word (ὄ ∷ χ ∷ ∙λ ∷ ο ∷ ς ∷ []) "John.6.5"
∷ word (ἔ ∷ ρ ∷ χ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.6.5"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.6.5"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.6.5"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.6.5"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.6.5"
∷ word (Φ ∷ ί ∷ ∙λ ∷ ι ∷ π ∷ π ∷ ο ∷ ν ∷ []) "John.6.5"
∷ word (Π ∷ ό ∷ θ ∷ ε ∷ ν ∷ []) "John.6.5"
∷ word (ἀ ∷ γ ∷ ο ∷ ρ ∷ ά ∷ σ ∷ ω ∷ μ ∷ ε ∷ ν ∷ []) "John.6.5"
∷ word (ἄ ∷ ρ ∷ τ ∷ ο ∷ υ ∷ ς ∷ []) "John.6.5"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.6.5"
∷ word (φ ∷ ά ∷ γ ∷ ω ∷ σ ∷ ι ∷ ν ∷ []) "John.6.5"
∷ word (ο ∷ ὗ ∷ τ ∷ ο ∷ ι ∷ []) "John.6.5"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.6.6"
∷ word (δ ∷ ὲ ∷ []) "John.6.6"
∷ word (ἔ ∷ ∙λ ∷ ε ∷ γ ∷ ε ∷ ν ∷ []) "John.6.6"
∷ word (π ∷ ε ∷ ι ∷ ρ ∷ ά ∷ ζ ∷ ω ∷ ν ∷ []) "John.6.6"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.6.6"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ς ∷ []) "John.6.6"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.6.6"
∷ word (ᾔ ∷ δ ∷ ε ∷ ι ∷ []) "John.6.6"
∷ word (τ ∷ ί ∷ []) "John.6.6"
∷ word (ἔ ∷ μ ∷ ε ∷ ∙λ ∷ ∙λ ∷ ε ∷ ν ∷ []) "John.6.6"
∷ word (π ∷ ο ∷ ι ∷ ε ∷ ῖ ∷ ν ∷ []) "John.6.6"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.6.7"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.6.7"
∷ word (Φ ∷ ί ∷ ∙λ ∷ ι ∷ π ∷ π ∷ ο ∷ ς ∷ []) "John.6.7"
∷ word (Δ ∷ ι ∷ α ∷ κ ∷ ο ∷ σ ∷ ί ∷ ω ∷ ν ∷ []) "John.6.7"
∷ word (δ ∷ η ∷ ν ∷ α ∷ ρ ∷ ί ∷ ω ∷ ν ∷ []) "John.6.7"
∷ word (ἄ ∷ ρ ∷ τ ∷ ο ∷ ι ∷ []) "John.6.7"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.6.7"
∷ word (ἀ ∷ ρ ∷ κ ∷ ο ∷ ῦ ∷ σ ∷ ι ∷ ν ∷ []) "John.6.7"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.6.7"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.6.7"
∷ word (ἕ ∷ κ ∷ α ∷ σ ∷ τ ∷ ο ∷ ς ∷ []) "John.6.7"
∷ word (β ∷ ρ ∷ α ∷ χ ∷ ύ ∷ []) "John.6.7"
∷ word (τ ∷ ι ∷ []) "John.6.7"
∷ word (∙λ ∷ ά ∷ β ∷ ῃ ∷ []) "John.6.7"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.6.8"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.6.8"
∷ word (ε ∷ ἷ ∷ ς ∷ []) "John.6.8"
∷ word (ἐ ∷ κ ∷ []) "John.6.8"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.6.8"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ ῶ ∷ ν ∷ []) "John.6.8"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.6.8"
∷ word (Ἀ ∷ ν ∷ δ ∷ ρ ∷ έ ∷ α ∷ ς ∷ []) "John.6.8"
∷ word (ὁ ∷ []) "John.6.8"
∷ word (ἀ ∷ δ ∷ ε ∷ ∙λ ∷ φ ∷ ὸ ∷ ς ∷ []) "John.6.8"
∷ word (Σ ∷ ί ∷ μ ∷ ω ∷ ν ∷ ο ∷ ς ∷ []) "John.6.8"
∷ word (Π ∷ έ ∷ τ ∷ ρ ∷ ο ∷ υ ∷ []) "John.6.8"
∷ word (Ἔ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.6.9"
∷ word (π ∷ α ∷ ι ∷ δ ∷ ά ∷ ρ ∷ ι ∷ ο ∷ ν ∷ []) "John.6.9"
∷ word (ὧ ∷ δ ∷ ε ∷ []) "John.6.9"
∷ word (ὃ ∷ ς ∷ []) "John.6.9"
∷ word (ἔ ∷ χ ∷ ε ∷ ι ∷ []) "John.6.9"
∷ word (π ∷ έ ∷ ν ∷ τ ∷ ε ∷ []) "John.6.9"
∷ word (ἄ ∷ ρ ∷ τ ∷ ο ∷ υ ∷ ς ∷ []) "John.6.9"
∷ word (κ ∷ ρ ∷ ι ∷ θ ∷ ί ∷ ν ∷ ο ∷ υ ∷ ς ∷ []) "John.6.9"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.6.9"
∷ word (δ ∷ ύ ∷ ο ∷ []) "John.6.9"
∷ word (ὀ ∷ ψ ∷ ά ∷ ρ ∷ ι ∷ α ∷ []) "John.6.9"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.6.9"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.6.9"
∷ word (τ ∷ ί ∷ []) "John.6.9"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.6.9"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.6.9"
∷ word (τ ∷ ο ∷ σ ∷ ο ∷ ύ ∷ τ ∷ ο ∷ υ ∷ ς ∷ []) "John.6.9"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.6.10"
∷ word (ὁ ∷ []) "John.6.10"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.6.10"
∷ word (Π ∷ ο ∷ ι ∷ ή ∷ σ ∷ α ∷ τ ∷ ε ∷ []) "John.6.10"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.6.10"
∷ word (ἀ ∷ ν ∷ θ ∷ ρ ∷ ώ ∷ π ∷ ο ∷ υ ∷ ς ∷ []) "John.6.10"
∷ word (ἀ ∷ ν ∷ α ∷ π ∷ ε ∷ σ ∷ ε ∷ ῖ ∷ ν ∷ []) "John.6.10"
∷ word (ἦ ∷ ν ∷ []) "John.6.10"
∷ word (δ ∷ ὲ ∷ []) "John.6.10"
∷ word (χ ∷ ό ∷ ρ ∷ τ ∷ ο ∷ ς ∷ []) "John.6.10"
∷ word (π ∷ ο ∷ ∙λ ∷ ὺ ∷ ς ∷ []) "John.6.10"
∷ word (ἐ ∷ ν ∷ []) "John.6.10"
∷ word (τ ∷ ῷ ∷ []) "John.6.10"
∷ word (τ ∷ ό ∷ π ∷ ῳ ∷ []) "John.6.10"
∷ word (ἀ ∷ ν ∷ έ ∷ π ∷ ε ∷ σ ∷ α ∷ ν ∷ []) "John.6.10"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.6.10"
∷ word (ο ∷ ἱ ∷ []) "John.6.10"
∷ word (ἄ ∷ ν ∷ δ ∷ ρ ∷ ε ∷ ς ∷ []) "John.6.10"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.6.10"
∷ word (ἀ ∷ ρ ∷ ι ∷ θ ∷ μ ∷ ὸ ∷ ν ∷ []) "John.6.10"
∷ word (ὡ ∷ ς ∷ []) "John.6.10"
∷ word (π ∷ ε ∷ ν ∷ τ ∷ α ∷ κ ∷ ι ∷ σ ∷ χ ∷ ί ∷ ∙λ ∷ ι ∷ ο ∷ ι ∷ []) "John.6.10"
∷ word (ἔ ∷ ∙λ ∷ α ∷ β ∷ ε ∷ ν ∷ []) "John.6.11"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.6.11"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.6.11"
∷ word (ἄ ∷ ρ ∷ τ ∷ ο ∷ υ ∷ ς ∷ []) "John.6.11"
∷ word (ὁ ∷ []) "John.6.11"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.6.11"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.6.11"
∷ word (ε ∷ ὐ ∷ χ ∷ α ∷ ρ ∷ ι ∷ σ ∷ τ ∷ ή ∷ σ ∷ α ∷ ς ∷ []) "John.6.11"
∷ word (δ ∷ ι ∷ έ ∷ δ ∷ ω ∷ κ ∷ ε ∷ ν ∷ []) "John.6.11"
∷ word (τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.6.11"
∷ word (ἀ ∷ ν ∷ α ∷ κ ∷ ε ∷ ι ∷ μ ∷ έ ∷ ν ∷ ο ∷ ι ∷ ς ∷ []) "John.6.11"
∷ word (ὁ ∷ μ ∷ ο ∷ ί ∷ ω ∷ ς ∷ []) "John.6.11"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.6.11"
∷ word (ἐ ∷ κ ∷ []) "John.6.11"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.6.11"
∷ word (ὀ ∷ ψ ∷ α ∷ ρ ∷ ί ∷ ω ∷ ν ∷ []) "John.6.11"
∷ word (ὅ ∷ σ ∷ ο ∷ ν ∷ []) "John.6.11"
∷ word (ἤ ∷ θ ∷ ε ∷ ∙λ ∷ ο ∷ ν ∷ []) "John.6.11"
∷ word (ὡ ∷ ς ∷ []) "John.6.12"
∷ word (δ ∷ ὲ ∷ []) "John.6.12"
∷ word (ἐ ∷ ν ∷ ε ∷ π ∷ ∙λ ∷ ή ∷ σ ∷ θ ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.6.12"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.6.12"
∷ word (τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.6.12"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ α ∷ ῖ ∷ ς ∷ []) "John.6.12"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.6.12"
∷ word (Σ ∷ υ ∷ ν ∷ α ∷ γ ∷ ά ∷ γ ∷ ε ∷ τ ∷ ε ∷ []) "John.6.12"
∷ word (τ ∷ ὰ ∷ []) "John.6.12"
∷ word (π ∷ ε ∷ ρ ∷ ι ∷ σ ∷ σ ∷ ε ∷ ύ ∷ σ ∷ α ∷ ν ∷ τ ∷ α ∷ []) "John.6.12"
∷ word (κ ∷ ∙λ ∷ ά ∷ σ ∷ μ ∷ α ∷ τ ∷ α ∷ []) "John.6.12"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.6.12"
∷ word (μ ∷ ή ∷ []) "John.6.12"
∷ word (τ ∷ ι ∷ []) "John.6.12"
∷ word (ἀ ∷ π ∷ ό ∷ ∙λ ∷ η ∷ τ ∷ α ∷ ι ∷ []) "John.6.12"
∷ word (σ ∷ υ ∷ ν ∷ ή ∷ γ ∷ α ∷ γ ∷ ο ∷ ν ∷ []) "John.6.13"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.6.13"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.6.13"
∷ word (ἐ ∷ γ ∷ έ ∷ μ ∷ ι ∷ σ ∷ α ∷ ν ∷ []) "John.6.13"
∷ word (δ ∷ ώ ∷ δ ∷ ε ∷ κ ∷ α ∷ []) "John.6.13"
∷ word (κ ∷ ο ∷ φ ∷ ί ∷ ν ∷ ο ∷ υ ∷ ς ∷ []) "John.6.13"
∷ word (κ ∷ ∙λ ∷ α ∷ σ ∷ μ ∷ ά ∷ τ ∷ ω ∷ ν ∷ []) "John.6.13"
∷ word (ἐ ∷ κ ∷ []) "John.6.13"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.6.13"
∷ word (π ∷ έ ∷ ν ∷ τ ∷ ε ∷ []) "John.6.13"
∷ word (ἄ ∷ ρ ∷ τ ∷ ω ∷ ν ∷ []) "John.6.13"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.6.13"
∷ word (κ ∷ ρ ∷ ι ∷ θ ∷ ί ∷ ν ∷ ω ∷ ν ∷ []) "John.6.13"
∷ word (ἃ ∷ []) "John.6.13"
∷ word (ἐ ∷ π ∷ ε ∷ ρ ∷ ί ∷ σ ∷ σ ∷ ε ∷ υ ∷ σ ∷ α ∷ ν ∷ []) "John.6.13"
∷ word (τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.6.13"
∷ word (β ∷ ε ∷ β ∷ ρ ∷ ω ∷ κ ∷ ό ∷ σ ∷ ι ∷ ν ∷ []) "John.6.13"
∷ word (ο ∷ ἱ ∷ []) "John.6.14"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.6.14"
∷ word (ἄ ∷ ν ∷ θ ∷ ρ ∷ ω ∷ π ∷ ο ∷ ι ∷ []) "John.6.14"
∷ word (ἰ ∷ δ ∷ ό ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.6.14"
∷ word (ὃ ∷ []) "John.6.14"
∷ word (ἐ ∷ π ∷ ο ∷ ί ∷ η ∷ σ ∷ ε ∷ ν ∷ []) "John.6.14"
∷ word (σ ∷ η ∷ μ ∷ ε ∷ ῖ ∷ ο ∷ ν ∷ []) "John.6.14"
∷ word (ἔ ∷ ∙λ ∷ ε ∷ γ ∷ ο ∷ ν ∷ []) "John.6.14"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.6.14"
∷ word (Ο ∷ ὗ ∷ τ ∷ ό ∷ ς ∷ []) "John.6.14"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.6.14"
∷ word (ἀ ∷ ∙λ ∷ η ∷ θ ∷ ῶ ∷ ς ∷ []) "John.6.14"
∷ word (ὁ ∷ []) "John.6.14"
∷ word (π ∷ ρ ∷ ο ∷ φ ∷ ή ∷ τ ∷ η ∷ ς ∷ []) "John.6.14"
∷ word (ὁ ∷ []) "John.6.14"
∷ word (ἐ ∷ ρ ∷ χ ∷ ό ∷ μ ∷ ε ∷ ν ∷ ο ∷ ς ∷ []) "John.6.14"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.6.14"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.6.14"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ ν ∷ []) "John.6.14"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.6.15"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.6.15"
∷ word (γ ∷ ν ∷ ο ∷ ὺ ∷ ς ∷ []) "John.6.15"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.6.15"
∷ word (μ ∷ έ ∷ ∙λ ∷ ∙λ ∷ ο ∷ υ ∷ σ ∷ ι ∷ ν ∷ []) "John.6.15"
∷ word (ἔ ∷ ρ ∷ χ ∷ ε ∷ σ ∷ θ ∷ α ∷ ι ∷ []) "John.6.15"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.6.15"
∷ word (ἁ ∷ ρ ∷ π ∷ ά ∷ ζ ∷ ε ∷ ι ∷ ν ∷ []) "John.6.15"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.6.15"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.6.15"
∷ word (π ∷ ο ∷ ι ∷ ή ∷ σ ∷ ω ∷ σ ∷ ι ∷ ν ∷ []) "John.6.15"
∷ word (β ∷ α ∷ σ ∷ ι ∷ ∙λ ∷ έ ∷ α ∷ []) "John.6.15"
∷ word (ἀ ∷ ν ∷ ε ∷ χ ∷ ώ ∷ ρ ∷ η ∷ σ ∷ ε ∷ ν ∷ []) "John.6.15"
∷ word (π ∷ ά ∷ ∙λ ∷ ι ∷ ν ∷ []) "John.6.15"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.6.15"
∷ word (τ ∷ ὸ ∷ []) "John.6.15"
∷ word (ὄ ∷ ρ ∷ ο ∷ ς ∷ []) "John.6.15"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ς ∷ []) "John.6.15"
∷ word (μ ∷ ό ∷ ν ∷ ο ∷ ς ∷ []) "John.6.15"
∷ word (Ὡ ∷ ς ∷ []) "John.6.16"
∷ word (δ ∷ ὲ ∷ []) "John.6.16"
∷ word (ὀ ∷ ψ ∷ ί ∷ α ∷ []) "John.6.16"
∷ word (ἐ ∷ γ ∷ έ ∷ ν ∷ ε ∷ τ ∷ ο ∷ []) "John.6.16"
∷ word (κ ∷ α ∷ τ ∷ έ ∷ β ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.6.16"
∷ word (ο ∷ ἱ ∷ []) "John.6.16"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ α ∷ ὶ ∷ []) "John.6.16"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.6.16"
∷ word (ἐ ∷ π ∷ ὶ ∷ []) "John.6.16"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.6.16"
∷ word (θ ∷ ά ∷ ∙λ ∷ α ∷ σ ∷ σ ∷ α ∷ ν ∷ []) "John.6.16"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.6.17"
∷ word (ἐ ∷ μ ∷ β ∷ ά ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.6.17"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.6.17"
∷ word (π ∷ ∙λ ∷ ο ∷ ῖ ∷ ο ∷ ν ∷ []) "John.6.17"
∷ word (ἤ ∷ ρ ∷ χ ∷ ο ∷ ν ∷ τ ∷ ο ∷ []) "John.6.17"
∷ word (π ∷ έ ∷ ρ ∷ α ∷ ν ∷ []) "John.6.17"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.6.17"
∷ word (θ ∷ α ∷ ∙λ ∷ ά ∷ σ ∷ σ ∷ η ∷ ς ∷ []) "John.6.17"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.6.17"
∷ word (Κ ∷ α ∷ φ ∷ α ∷ ρ ∷ ν ∷ α ∷ ο ∷ ύ ∷ μ ∷ []) "John.6.17"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.6.17"
∷ word (σ ∷ κ ∷ ο ∷ τ ∷ ί ∷ α ∷ []) "John.6.17"
∷ word (ἤ ∷ δ ∷ η ∷ []) "John.6.17"
∷ word (ἐ ∷ γ ∷ ε ∷ γ ∷ ό ∷ ν ∷ ε ∷ ι ∷ []) "John.6.17"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.6.17"
∷ word (ο ∷ ὔ ∷ π ∷ ω ∷ []) "John.6.17"
∷ word (ἐ ∷ ∙λ ∷ η ∷ ∙λ ∷ ύ ∷ θ ∷ ε ∷ ι ∷ []) "John.6.17"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.6.17"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.6.17"
∷ word (ὁ ∷ []) "John.6.17"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.6.17"
∷ word (ἥ ∷ []) "John.6.18"
∷ word (τ ∷ ε ∷ []) "John.6.18"
∷ word (θ ∷ ά ∷ ∙λ ∷ α ∷ σ ∷ σ ∷ α ∷ []) "John.6.18"
∷ word (ἀ ∷ ν ∷ έ ∷ μ ∷ ο ∷ υ ∷ []) "John.6.18"
∷ word (μ ∷ ε ∷ γ ∷ ά ∷ ∙λ ∷ ο ∷ υ ∷ []) "John.6.18"
∷ word (π ∷ ν ∷ έ ∷ ο ∷ ν ∷ τ ∷ ο ∷ ς ∷ []) "John.6.18"
∷ word (δ ∷ ι ∷ ε ∷ γ ∷ ε ∷ ί ∷ ρ ∷ ε ∷ τ ∷ ο ∷ []) "John.6.18"
∷ word (ἐ ∷ ∙λ ∷ η ∷ ∙λ ∷ α ∷ κ ∷ ό ∷ τ ∷ ε ∷ ς ∷ []) "John.6.19"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.6.19"
∷ word (ὡ ∷ ς ∷ []) "John.6.19"
∷ word (σ ∷ τ ∷ α ∷ δ ∷ ί ∷ ο ∷ υ ∷ ς ∷ []) "John.6.19"
∷ word (ε ∷ ἴ ∷ κ ∷ ο ∷ σ ∷ ι ∷ []) "John.6.19"
∷ word (π ∷ έ ∷ ν ∷ τ ∷ ε ∷ []) "John.6.19"
∷ word (ἢ ∷ []) "John.6.19"
∷ word (τ ∷ ρ ∷ ι ∷ ά ∷ κ ∷ ο ∷ ν ∷ τ ∷ α ∷ []) "John.6.19"
∷ word (θ ∷ ε ∷ ω ∷ ρ ∷ ο ∷ ῦ ∷ σ ∷ ι ∷ ν ∷ []) "John.6.19"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.6.19"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ν ∷ []) "John.6.19"
∷ word (π ∷ ε ∷ ρ ∷ ι ∷ π ∷ α ∷ τ ∷ ο ∷ ῦ ∷ ν ∷ τ ∷ α ∷ []) "John.6.19"
∷ word (ἐ ∷ π ∷ ὶ ∷ []) "John.6.19"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.6.19"
∷ word (θ ∷ α ∷ ∙λ ∷ ά ∷ σ ∷ σ ∷ η ∷ ς ∷ []) "John.6.19"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.6.19"
∷ word (ἐ ∷ γ ∷ γ ∷ ὺ ∷ ς ∷ []) "John.6.19"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.6.19"
∷ word (π ∷ ∙λ ∷ ο ∷ ί ∷ ο ∷ υ ∷ []) "John.6.19"
∷ word (γ ∷ ι ∷ ν ∷ ό ∷ μ ∷ ε ∷ ν ∷ ο ∷ ν ∷ []) "John.6.19"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.6.19"
∷ word (ἐ ∷ φ ∷ ο ∷ β ∷ ή ∷ θ ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.6.19"
∷ word (ὁ ∷ []) "John.6.20"
∷ word (δ ∷ ὲ ∷ []) "John.6.20"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.6.20"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.6.20"
∷ word (Ἐ ∷ γ ∷ ώ ∷ []) "John.6.20"
∷ word (ε ∷ ἰ ∷ μ ∷ ι ∷ []) "John.6.20"
∷ word (μ ∷ ὴ ∷ []) "John.6.20"
∷ word (φ ∷ ο ∷ β ∷ ε ∷ ῖ ∷ σ ∷ θ ∷ ε ∷ []) "John.6.20"
∷ word (ἤ ∷ θ ∷ ε ∷ ∙λ ∷ ο ∷ ν ∷ []) "John.6.21"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.6.21"
∷ word (∙λ ∷ α ∷ β ∷ ε ∷ ῖ ∷ ν ∷ []) "John.6.21"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.6.21"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.6.21"
∷ word (τ ∷ ὸ ∷ []) "John.6.21"
∷ word (π ∷ ∙λ ∷ ο ∷ ῖ ∷ ο ∷ ν ∷ []) "John.6.21"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.6.21"
∷ word (ε ∷ ὐ ∷ θ ∷ έ ∷ ω ∷ ς ∷ []) "John.6.21"
∷ word (ἐ ∷ γ ∷ έ ∷ ν ∷ ε ∷ τ ∷ ο ∷ []) "John.6.21"
∷ word (τ ∷ ὸ ∷ []) "John.6.21"
∷ word (π ∷ ∙λ ∷ ο ∷ ῖ ∷ ο ∷ ν ∷ []) "John.6.21"
∷ word (ἐ ∷ π ∷ ὶ ∷ []) "John.6.21"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.6.21"
∷ word (γ ∷ ῆ ∷ ς ∷ []) "John.6.21"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.6.21"
∷ word (ἣ ∷ ν ∷ []) "John.6.21"
∷ word (ὑ ∷ π ∷ ῆ ∷ γ ∷ ο ∷ ν ∷ []) "John.6.21"
∷ word (Τ ∷ ῇ ∷ []) "John.6.22"
∷ word (ἐ ∷ π ∷ α ∷ ύ ∷ ρ ∷ ι ∷ ο ∷ ν ∷ []) "John.6.22"
∷ word (ὁ ∷ []) "John.6.22"
∷ word (ὄ ∷ χ ∷ ∙λ ∷ ο ∷ ς ∷ []) "John.6.22"
∷ word (ὁ ∷ []) "John.6.22"
∷ word (ἑ ∷ σ ∷ τ ∷ η ∷ κ ∷ ὼ ∷ ς ∷ []) "John.6.22"
∷ word (π ∷ έ ∷ ρ ∷ α ∷ ν ∷ []) "John.6.22"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.6.22"
∷ word (θ ∷ α ∷ ∙λ ∷ ά ∷ σ ∷ σ ∷ η ∷ ς ∷ []) "John.6.22"
∷ word (ε ∷ ἶ ∷ δ ∷ ο ∷ ν ∷ []) "John.6.22"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.6.22"
∷ word (π ∷ ∙λ ∷ ο ∷ ι ∷ ά ∷ ρ ∷ ι ∷ ο ∷ ν ∷ []) "John.6.22"
∷ word (ἄ ∷ ∙λ ∷ ∙λ ∷ ο ∷ []) "John.6.22"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.6.22"
∷ word (ἦ ∷ ν ∷ []) "John.6.22"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ []) "John.6.22"
∷ word (ε ∷ ἰ ∷ []) "John.6.22"
∷ word (μ ∷ ὴ ∷ []) "John.6.22"
∷ word (ἕ ∷ ν ∷ []) "John.6.22"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.6.22"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.6.22"
∷ word (ο ∷ ὐ ∷ []) "John.6.22"
∷ word (σ ∷ υ ∷ ν ∷ ε ∷ ι ∷ σ ∷ ῆ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.6.22"
∷ word (τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.6.22"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ α ∷ ῖ ∷ ς ∷ []) "John.6.22"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.6.22"
∷ word (ὁ ∷ []) "John.6.22"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.6.22"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.6.22"
∷ word (τ ∷ ὸ ∷ []) "John.6.22"
∷ word (π ∷ ∙λ ∷ ο ∷ ῖ ∷ ο ∷ ν ∷ []) "John.6.22"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.6.22"
∷ word (μ ∷ ό ∷ ν ∷ ο ∷ ι ∷ []) "John.6.22"
∷ word (ο ∷ ἱ ∷ []) "John.6.22"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ α ∷ ὶ ∷ []) "John.6.22"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.6.22"
∷ word (ἀ ∷ π ∷ ῆ ∷ ∙λ ∷ θ ∷ ο ∷ ν ∷ []) "John.6.22"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.6.23"
∷ word (ἦ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.6.23"
∷ word (π ∷ ∙λ ∷ ο ∷ ι ∷ ά ∷ ρ ∷ ι ∷ α ∷ []) "John.6.23"
∷ word (ἐ ∷ κ ∷ []) "John.6.23"
∷ word (Τ ∷ ι ∷ β ∷ ε ∷ ρ ∷ ι ∷ ά ∷ δ ∷ ο ∷ ς ∷ []) "John.6.23"
∷ word (ἐ ∷ γ ∷ γ ∷ ὺ ∷ ς ∷ []) "John.6.23"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.6.23"
∷ word (τ ∷ ό ∷ π ∷ ο ∷ υ ∷ []) "John.6.23"
∷ word (ὅ ∷ π ∷ ο ∷ υ ∷ []) "John.6.23"
∷ word (ἔ ∷ φ ∷ α ∷ γ ∷ ο ∷ ν ∷ []) "John.6.23"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.6.23"
∷ word (ἄ ∷ ρ ∷ τ ∷ ο ∷ ν ∷ []) "John.6.23"
∷ word (ε ∷ ὐ ∷ χ ∷ α ∷ ρ ∷ ι ∷ σ ∷ τ ∷ ή ∷ σ ∷ α ∷ ν ∷ τ ∷ ο ∷ ς ∷ []) "John.6.23"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.6.23"
∷ word (κ ∷ υ ∷ ρ ∷ ί ∷ ο ∷ υ ∷ []) "John.6.23"
∷ word (ὅ ∷ τ ∷ ε ∷ []) "John.6.24"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.6.24"
∷ word (ε ∷ ἶ ∷ δ ∷ ε ∷ ν ∷ []) "John.6.24"
∷ word (ὁ ∷ []) "John.6.24"
∷ word (ὄ ∷ χ ∷ ∙λ ∷ ο ∷ ς ∷ []) "John.6.24"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.6.24"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.6.24"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.6.24"
∷ word (ἔ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.6.24"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ []) "John.6.24"
∷ word (ο ∷ ὐ ∷ δ ∷ ὲ ∷ []) "John.6.24"
∷ word (ο ∷ ἱ ∷ []) "John.6.24"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ α ∷ ὶ ∷ []) "John.6.24"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.6.24"
∷ word (ἐ ∷ ν ∷ έ ∷ β ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.6.24"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ὶ ∷ []) "John.6.24"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.6.24"
∷ word (τ ∷ ὰ ∷ []) "John.6.24"
∷ word (π ∷ ∙λ ∷ ο ∷ ι ∷ ά ∷ ρ ∷ ι ∷ α ∷ []) "John.6.24"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.6.24"
∷ word (ἦ ∷ ∙λ ∷ θ ∷ ο ∷ ν ∷ []) "John.6.24"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.6.24"
∷ word (Κ ∷ α ∷ φ ∷ α ∷ ρ ∷ ν ∷ α ∷ ο ∷ ὺ ∷ μ ∷ []) "John.6.24"
∷ word (ζ ∷ η ∷ τ ∷ ο ∷ ῦ ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.6.24"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.6.24"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ν ∷ []) "John.6.24"
∷ word (Κ ∷ α ∷ ὶ ∷ []) "John.6.25"
∷ word (ε ∷ ὑ ∷ ρ ∷ ό ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.6.25"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.6.25"
∷ word (π ∷ έ ∷ ρ ∷ α ∷ ν ∷ []) "John.6.25"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.6.25"
∷ word (θ ∷ α ∷ ∙λ ∷ ά ∷ σ ∷ σ ∷ η ∷ ς ∷ []) "John.6.25"
∷ word (ε ∷ ἶ ∷ π ∷ ο ∷ ν ∷ []) "John.6.25"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.6.25"
∷ word (Ῥ ∷ α ∷ β ∷ β ∷ ί ∷ []) "John.6.25"
∷ word (π ∷ ό ∷ τ ∷ ε ∷ []) "John.6.25"
∷ word (ὧ ∷ δ ∷ ε ∷ []) "John.6.25"
∷ word (γ ∷ έ ∷ γ ∷ ο ∷ ν ∷ α ∷ ς ∷ []) "John.6.25"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.6.26"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.6.26"
∷ word (ὁ ∷ []) "John.6.26"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.6.26"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.6.26"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.6.26"
∷ word (Ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.6.26"
∷ word (ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.6.26"
∷ word (∙λ ∷ έ ∷ γ ∷ ω ∷ []) "John.6.26"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.6.26"
∷ word (ζ ∷ η ∷ τ ∷ ε ∷ ῖ ∷ τ ∷ έ ∷ []) "John.6.26"
∷ word (μ ∷ ε ∷ []) "John.6.26"
∷ word (ο ∷ ὐ ∷ χ ∷ []) "John.6.26"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.6.26"
∷ word (ε ∷ ἴ ∷ δ ∷ ε ∷ τ ∷ ε ∷ []) "John.6.26"
∷ word (σ ∷ η ∷ μ ∷ ε ∷ ῖ ∷ α ∷ []) "John.6.26"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ []) "John.6.26"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.6.26"
∷ word (ἐ ∷ φ ∷ ά ∷ γ ∷ ε ∷ τ ∷ ε ∷ []) "John.6.26"
∷ word (ἐ ∷ κ ∷ []) "John.6.26"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.6.26"
∷ word (ἄ ∷ ρ ∷ τ ∷ ω ∷ ν ∷ []) "John.6.26"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.6.26"
∷ word (ἐ ∷ χ ∷ ο ∷ ρ ∷ τ ∷ ά ∷ σ ∷ θ ∷ η ∷ τ ∷ ε ∷ []) "John.6.26"
∷ word (ἐ ∷ ρ ∷ γ ∷ ά ∷ ζ ∷ ε ∷ σ ∷ θ ∷ ε ∷ []) "John.6.27"
∷ word (μ ∷ ὴ ∷ []) "John.6.27"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.6.27"
∷ word (β ∷ ρ ∷ ῶ ∷ σ ∷ ι ∷ ν ∷ []) "John.6.27"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.6.27"
∷ word (ἀ ∷ π ∷ ο ∷ ∙λ ∷ ∙λ ∷ υ ∷ μ ∷ έ ∷ ν ∷ η ∷ ν ∷ []) "John.6.27"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.6.27"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.6.27"
∷ word (β ∷ ρ ∷ ῶ ∷ σ ∷ ι ∷ ν ∷ []) "John.6.27"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.6.27"
∷ word (μ ∷ έ ∷ ν ∷ ο ∷ υ ∷ σ ∷ α ∷ ν ∷ []) "John.6.27"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.6.27"
∷ word (ζ ∷ ω ∷ ὴ ∷ ν ∷ []) "John.6.27"
∷ word (α ∷ ἰ ∷ ώ ∷ ν ∷ ι ∷ ο ∷ ν ∷ []) "John.6.27"
∷ word (ἣ ∷ ν ∷ []) "John.6.27"
∷ word (ὁ ∷ []) "John.6.27"
∷ word (υ ∷ ἱ ∷ ὸ ∷ ς ∷ []) "John.6.27"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.6.27"
∷ word (ἀ ∷ ν ∷ θ ∷ ρ ∷ ώ ∷ π ∷ ο ∷ υ ∷ []) "John.6.27"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.6.27"
∷ word (δ ∷ ώ ∷ σ ∷ ε ∷ ι ∷ []) "John.6.27"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ ν ∷ []) "John.6.27"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.6.27"
∷ word (ὁ ∷ []) "John.6.27"
∷ word (π ∷ α ∷ τ ∷ ὴ ∷ ρ ∷ []) "John.6.27"
∷ word (ἐ ∷ σ ∷ φ ∷ ρ ∷ ά ∷ γ ∷ ι ∷ σ ∷ ε ∷ ν ∷ []) "John.6.27"
∷ word (ὁ ∷ []) "John.6.27"
∷ word (θ ∷ ε ∷ ό ∷ ς ∷ []) "John.6.27"
∷ word (ε ∷ ἶ ∷ π ∷ ο ∷ ν ∷ []) "John.6.28"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.6.28"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.6.28"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.6.28"
∷ word (Τ ∷ ί ∷ []) "John.6.28"
∷ word (π ∷ ο ∷ ι ∷ ῶ ∷ μ ∷ ε ∷ ν ∷ []) "John.6.28"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.6.28"
∷ word (ἐ ∷ ρ ∷ γ ∷ α ∷ ζ ∷ ώ ∷ μ ∷ ε ∷ θ ∷ α ∷ []) "John.6.28"
∷ word (τ ∷ ὰ ∷ []) "John.6.28"
∷ word (ἔ ∷ ρ ∷ γ ∷ α ∷ []) "John.6.28"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.6.28"
∷ word (θ ∷ ε ∷ ο ∷ ῦ ∷ []) "John.6.28"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.6.29"
∷ word (ὁ ∷ []) "John.6.29"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.6.29"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.6.29"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.6.29"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.6.29"
∷ word (Τ ∷ ο ∷ ῦ ∷ τ ∷ ό ∷ []) "John.6.29"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.6.29"
∷ word (τ ∷ ὸ ∷ []) "John.6.29"
∷ word (ἔ ∷ ρ ∷ γ ∷ ο ∷ ν ∷ []) "John.6.29"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.6.29"
∷ word (θ ∷ ε ∷ ο ∷ ῦ ∷ []) "John.6.29"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.6.29"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ η ∷ τ ∷ ε ∷ []) "John.6.29"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.6.29"
∷ word (ὃ ∷ ν ∷ []) "John.6.29"
∷ word (ἀ ∷ π ∷ έ ∷ σ ∷ τ ∷ ε ∷ ι ∷ ∙λ ∷ ε ∷ ν ∷ []) "John.6.29"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ο ∷ ς ∷ []) "John.6.29"
∷ word (ε ∷ ἶ ∷ π ∷ ο ∷ ν ∷ []) "John.6.30"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.6.30"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.6.30"
∷ word (Τ ∷ ί ∷ []) "John.6.30"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.6.30"
∷ word (π ∷ ο ∷ ι ∷ ε ∷ ῖ ∷ ς ∷ []) "John.6.30"
∷ word (σ ∷ ὺ ∷ []) "John.6.30"
∷ word (σ ∷ η ∷ μ ∷ ε ∷ ῖ ∷ ο ∷ ν ∷ []) "John.6.30"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.6.30"
∷ word (ἴ ∷ δ ∷ ω ∷ μ ∷ ε ∷ ν ∷ []) "John.6.30"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.6.30"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ σ ∷ ω ∷ μ ∷ έ ∷ ν ∷ []) "John.6.30"
∷ word (σ ∷ ο ∷ ι ∷ []) "John.6.30"
∷ word (τ ∷ ί ∷ []) "John.6.30"
∷ word (ἐ ∷ ρ ∷ γ ∷ ά ∷ ζ ∷ ῃ ∷ []) "John.6.30"
∷ word (ο ∷ ἱ ∷ []) "John.6.31"
∷ word (π ∷ α ∷ τ ∷ έ ∷ ρ ∷ ε ∷ ς ∷ []) "John.6.31"
∷ word (ἡ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.6.31"
∷ word (τ ∷ ὸ ∷ []) "John.6.31"
∷ word (μ ∷ ά ∷ ν ∷ ν ∷ α ∷ []) "John.6.31"
∷ word (ἔ ∷ φ ∷ α ∷ γ ∷ ο ∷ ν ∷ []) "John.6.31"
∷ word (ἐ ∷ ν ∷ []) "John.6.31"
∷ word (τ ∷ ῇ ∷ []) "John.6.31"
∷ word (ἐ ∷ ρ ∷ ή ∷ μ ∷ ῳ ∷ []) "John.6.31"
∷ word (κ ∷ α ∷ θ ∷ ώ ∷ ς ∷ []) "John.6.31"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.6.31"
∷ word (γ ∷ ε ∷ γ ∷ ρ ∷ α ∷ μ ∷ μ ∷ έ ∷ ν ∷ ο ∷ ν ∷ []) "John.6.31"
∷ word (Ἄ ∷ ρ ∷ τ ∷ ο ∷ ν ∷ []) "John.6.31"
∷ word (ἐ ∷ κ ∷ []) "John.6.31"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.6.31"
∷ word (ο ∷ ὐ ∷ ρ ∷ α ∷ ν ∷ ο ∷ ῦ ∷ []) "John.6.31"
∷ word (ἔ ∷ δ ∷ ω ∷ κ ∷ ε ∷ ν ∷ []) "John.6.31"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.6.31"
∷ word (φ ∷ α ∷ γ ∷ ε ∷ ῖ ∷ ν ∷ []) "John.6.31"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.6.32"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.6.32"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.6.32"
∷ word (ὁ ∷ []) "John.6.32"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.6.32"
∷ word (Ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.6.32"
∷ word (ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.6.32"
∷ word (∙λ ∷ έ ∷ γ ∷ ω ∷ []) "John.6.32"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.6.32"
∷ word (ο ∷ ὐ ∷ []) "John.6.32"
∷ word (Μ ∷ ω ∷ ϋ ∷ σ ∷ ῆ ∷ ς ∷ []) "John.6.32"
∷ word (δ ∷ έ ∷ δ ∷ ω ∷ κ ∷ ε ∷ ν ∷ []) "John.6.32"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.6.32"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.6.32"
∷ word (ἄ ∷ ρ ∷ τ ∷ ο ∷ ν ∷ []) "John.6.32"
∷ word (ἐ ∷ κ ∷ []) "John.6.32"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.6.32"
∷ word (ο ∷ ὐ ∷ ρ ∷ α ∷ ν ∷ ο ∷ ῦ ∷ []) "John.6.32"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ []) "John.6.32"
∷ word (ὁ ∷ []) "John.6.32"
∷ word (π ∷ α ∷ τ ∷ ή ∷ ρ ∷ []) "John.6.32"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.6.32"
∷ word (δ ∷ ί ∷ δ ∷ ω ∷ σ ∷ ι ∷ ν ∷ []) "John.6.32"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.6.32"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.6.32"
∷ word (ἄ ∷ ρ ∷ τ ∷ ο ∷ ν ∷ []) "John.6.32"
∷ word (ἐ ∷ κ ∷ []) "John.6.32"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.6.32"
∷ word (ο ∷ ὐ ∷ ρ ∷ α ∷ ν ∷ ο ∷ ῦ ∷ []) "John.6.32"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.6.32"
∷ word (ἀ ∷ ∙λ ∷ η ∷ θ ∷ ι ∷ ν ∷ ό ∷ ν ∷ []) "John.6.32"
∷ word (ὁ ∷ []) "John.6.33"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.6.33"
∷ word (ἄ ∷ ρ ∷ τ ∷ ο ∷ ς ∷ []) "John.6.33"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.6.33"
∷ word (θ ∷ ε ∷ ο ∷ ῦ ∷ []) "John.6.33"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.6.33"
∷ word (ὁ ∷ []) "John.6.33"
∷ word (κ ∷ α ∷ τ ∷ α ∷ β ∷ α ∷ ί ∷ ν ∷ ω ∷ ν ∷ []) "John.6.33"
∷ word (ἐ ∷ κ ∷ []) "John.6.33"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.6.33"
∷ word (ο ∷ ὐ ∷ ρ ∷ α ∷ ν ∷ ο ∷ ῦ ∷ []) "John.6.33"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.6.33"
∷ word (ζ ∷ ω ∷ ὴ ∷ ν ∷ []) "John.6.33"
∷ word (δ ∷ ι ∷ δ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.6.33"
∷ word (τ ∷ ῷ ∷ []) "John.6.33"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ῳ ∷ []) "John.6.33"
∷ word (ε ∷ ἶ ∷ π ∷ ο ∷ ν ∷ []) "John.6.34"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.6.34"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.6.34"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.6.34"
∷ word (Κ ∷ ύ ∷ ρ ∷ ι ∷ ε ∷ []) "John.6.34"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ ο ∷ τ ∷ ε ∷ []) "John.6.34"
∷ word (δ ∷ ὸ ∷ ς ∷ []) "John.6.34"
∷ word (ἡ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.6.34"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.6.34"
∷ word (ἄ ∷ ρ ∷ τ ∷ ο ∷ ν ∷ []) "John.6.34"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ ν ∷ []) "John.6.34"
∷ word (Ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.6.35"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.6.35"
∷ word (ὁ ∷ []) "John.6.35"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.6.35"
∷ word (Ἐ ∷ γ ∷ ώ ∷ []) "John.6.35"
∷ word (ε ∷ ἰ ∷ μ ∷ ι ∷ []) "John.6.35"
∷ word (ὁ ∷ []) "John.6.35"
∷ word (ἄ ∷ ρ ∷ τ ∷ ο ∷ ς ∷ []) "John.6.35"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.6.35"
∷ word (ζ ∷ ω ∷ ῆ ∷ ς ∷ []) "John.6.35"
∷ word (ὁ ∷ []) "John.6.35"
∷ word (ἐ ∷ ρ ∷ χ ∷ ό ∷ μ ∷ ε ∷ ν ∷ ο ∷ ς ∷ []) "John.6.35"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.6.35"
∷ word (ἐ ∷ μ ∷ ὲ ∷ []) "John.6.35"
∷ word (ο ∷ ὐ ∷ []) "John.6.35"
∷ word (μ ∷ ὴ ∷ []) "John.6.35"
∷ word (π ∷ ε ∷ ι ∷ ν ∷ ά ∷ σ ∷ ῃ ∷ []) "John.6.35"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.6.35"
∷ word (ὁ ∷ []) "John.6.35"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ ω ∷ ν ∷ []) "John.6.35"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.6.35"
∷ word (ἐ ∷ μ ∷ ὲ ∷ []) "John.6.35"
∷ word (ο ∷ ὐ ∷ []) "John.6.35"
∷ word (μ ∷ ὴ ∷ []) "John.6.35"
∷ word (δ ∷ ι ∷ ψ ∷ ή ∷ σ ∷ ε ∷ ι ∷ []) "John.6.35"
∷ word (π ∷ ώ ∷ π ∷ ο ∷ τ ∷ ε ∷ []) "John.6.35"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ []) "John.6.36"
∷ word (ε ∷ ἶ ∷ π ∷ ο ∷ ν ∷ []) "John.6.36"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.6.36"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.6.36"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.6.36"
∷ word (ἑ ∷ ω ∷ ρ ∷ ά ∷ κ ∷ α ∷ τ ∷ έ ∷ []) "John.6.36"
∷ word (μ ∷ ε ∷ []) "John.6.36"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.6.36"
∷ word (ο ∷ ὐ ∷ []) "John.6.36"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ ε ∷ τ ∷ ε ∷ []) "John.6.36"
∷ word (π ∷ ᾶ ∷ ν ∷ []) "John.6.37"
∷ word (ὃ ∷ []) "John.6.37"
∷ word (δ ∷ ί ∷ δ ∷ ω ∷ σ ∷ ί ∷ ν ∷ []) "John.6.37"
∷ word (μ ∷ ο ∷ ι ∷ []) "John.6.37"
∷ word (ὁ ∷ []) "John.6.37"
∷ word (π ∷ α ∷ τ ∷ ὴ ∷ ρ ∷ []) "John.6.37"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.6.37"
∷ word (ἐ ∷ μ ∷ ὲ ∷ []) "John.6.37"
∷ word (ἥ ∷ ξ ∷ ε ∷ ι ∷ []) "John.6.37"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.6.37"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.6.37"
∷ word (ἐ ∷ ρ ∷ χ ∷ ό ∷ μ ∷ ε ∷ ν ∷ ο ∷ ν ∷ []) "John.6.37"
∷ word (π ∷ ρ ∷ ό ∷ ς ∷ []) "John.6.37"
∷ word (μ ∷ ε ∷ []) "John.6.37"
∷ word (ο ∷ ὐ ∷ []) "John.6.37"
∷ word (μ ∷ ὴ ∷ []) "John.6.37"
∷ word (ἐ ∷ κ ∷ β ∷ ά ∷ ∙λ ∷ ω ∷ []) "John.6.37"
∷ word (ἔ ∷ ξ ∷ ω ∷ []) "John.6.37"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.6.38"
∷ word (κ ∷ α ∷ τ ∷ α ∷ β ∷ έ ∷ β ∷ η ∷ κ ∷ α ∷ []) "John.6.38"
∷ word (ἀ ∷ π ∷ ὸ ∷ []) "John.6.38"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.6.38"
∷ word (ο ∷ ὐ ∷ ρ ∷ α ∷ ν ∷ ο ∷ ῦ ∷ []) "John.6.38"
∷ word (ο ∷ ὐ ∷ χ ∷ []) "John.6.38"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.6.38"
∷ word (π ∷ ο ∷ ι ∷ ῶ ∷ []) "John.6.38"
∷ word (τ ∷ ὸ ∷ []) "John.6.38"
∷ word (θ ∷ έ ∷ ∙λ ∷ η ∷ μ ∷ α ∷ []) "John.6.38"
∷ word (τ ∷ ὸ ∷ []) "John.6.38"
∷ word (ἐ ∷ μ ∷ ὸ ∷ ν ∷ []) "John.6.38"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.6.38"
∷ word (τ ∷ ὸ ∷ []) "John.6.38"
∷ word (θ ∷ έ ∷ ∙λ ∷ η ∷ μ ∷ α ∷ []) "John.6.38"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.6.38"
∷ word (π ∷ έ ∷ μ ∷ ψ ∷ α ∷ ν ∷ τ ∷ ό ∷ ς ∷ []) "John.6.38"
∷ word (μ ∷ ε ∷ []) "John.6.38"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.6.39"
∷ word (δ ∷ έ ∷ []) "John.6.39"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.6.39"
∷ word (τ ∷ ὸ ∷ []) "John.6.39"
∷ word (θ ∷ έ ∷ ∙λ ∷ η ∷ μ ∷ α ∷ []) "John.6.39"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.6.39"
∷ word (π ∷ έ ∷ μ ∷ ψ ∷ α ∷ ν ∷ τ ∷ ό ∷ ς ∷ []) "John.6.39"
∷ word (μ ∷ ε ∷ []) "John.6.39"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.6.39"
∷ word (π ∷ ᾶ ∷ ν ∷ []) "John.6.39"
∷ word (ὃ ∷ []) "John.6.39"
∷ word (δ ∷ έ ∷ δ ∷ ω ∷ κ ∷ έ ∷ ν ∷ []) "John.6.39"
∷ word (μ ∷ ο ∷ ι ∷ []) "John.6.39"
∷ word (μ ∷ ὴ ∷ []) "John.6.39"
∷ word (ἀ ∷ π ∷ ο ∷ ∙λ ∷ έ ∷ σ ∷ ω ∷ []) "John.6.39"
∷ word (ἐ ∷ ξ ∷ []) "John.6.39"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.6.39"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.6.39"
∷ word (ἀ ∷ ν ∷ α ∷ σ ∷ τ ∷ ή ∷ σ ∷ ω ∷ []) "John.6.39"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ []) "John.6.39"
∷ word (τ ∷ ῇ ∷ []) "John.6.39"
∷ word (ἐ ∷ σ ∷ χ ∷ ά ∷ τ ∷ ῃ ∷ []) "John.6.39"
∷ word (ἡ ∷ μ ∷ έ ∷ ρ ∷ ᾳ ∷ []) "John.6.39"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.6.40"
∷ word (γ ∷ ά ∷ ρ ∷ []) "John.6.40"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.6.40"
∷ word (τ ∷ ὸ ∷ []) "John.6.40"
∷ word (θ ∷ έ ∷ ∙λ ∷ η ∷ μ ∷ α ∷ []) "John.6.40"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.6.40"
∷ word (π ∷ α ∷ τ ∷ ρ ∷ ό ∷ ς ∷ []) "John.6.40"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.6.40"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.6.40"
∷ word (π ∷ ᾶ ∷ ς ∷ []) "John.6.40"
∷ word (ὁ ∷ []) "John.6.40"
∷ word (θ ∷ ε ∷ ω ∷ ρ ∷ ῶ ∷ ν ∷ []) "John.6.40"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.6.40"
∷ word (υ ∷ ἱ ∷ ὸ ∷ ν ∷ []) "John.6.40"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.6.40"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ ω ∷ ν ∷ []) "John.6.40"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.6.40"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.6.40"
∷ word (ἔ ∷ χ ∷ ῃ ∷ []) "John.6.40"
∷ word (ζ ∷ ω ∷ ὴ ∷ ν ∷ []) "John.6.40"
∷ word (α ∷ ἰ ∷ ώ ∷ ν ∷ ι ∷ ο ∷ ν ∷ []) "John.6.40"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.6.40"
∷ word (ἀ ∷ ν ∷ α ∷ σ ∷ τ ∷ ή ∷ σ ∷ ω ∷ []) "John.6.40"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.6.40"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.6.40"
∷ word (τ ∷ ῇ ∷ []) "John.6.40"
∷ word (ἐ ∷ σ ∷ χ ∷ ά ∷ τ ∷ ῃ ∷ []) "John.6.40"
∷ word (ἡ ∷ μ ∷ έ ∷ ρ ∷ ᾳ ∷ []) "John.6.40"
∷ word (Ἐ ∷ γ ∷ ό ∷ γ ∷ γ ∷ υ ∷ ζ ∷ ο ∷ ν ∷ []) "John.6.41"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.6.41"
∷ word (ο ∷ ἱ ∷ []) "John.6.41"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ῖ ∷ ο ∷ ι ∷ []) "John.6.41"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.6.41"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.6.41"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.6.41"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.6.41"
∷ word (Ἐ ∷ γ ∷ ώ ∷ []) "John.6.41"
∷ word (ε ∷ ἰ ∷ μ ∷ ι ∷ []) "John.6.41"
∷ word (ὁ ∷ []) "John.6.41"
∷ word (ἄ ∷ ρ ∷ τ ∷ ο ∷ ς ∷ []) "John.6.41"
∷ word (ὁ ∷ []) "John.6.41"
∷ word (κ ∷ α ∷ τ ∷ α ∷ β ∷ ὰ ∷ ς ∷ []) "John.6.41"
∷ word (ἐ ∷ κ ∷ []) "John.6.41"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.6.41"
∷ word (ο ∷ ὐ ∷ ρ ∷ α ∷ ν ∷ ο ∷ ῦ ∷ []) "John.6.41"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.6.42"
∷ word (ἔ ∷ ∙λ ∷ ε ∷ γ ∷ ο ∷ ν ∷ []) "John.6.42"
∷ word (Ο ∷ ὐ ∷ χ ∷ []) "John.6.42"
∷ word (ο ∷ ὗ ∷ τ ∷ ό ∷ ς ∷ []) "John.6.42"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.6.42"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.6.42"
∷ word (ὁ ∷ []) "John.6.42"
∷ word (υ ∷ ἱ ∷ ὸ ∷ ς ∷ []) "John.6.42"
∷ word (Ἰ ∷ ω ∷ σ ∷ ή ∷ φ ∷ []) "John.6.42"
∷ word (ο ∷ ὗ ∷ []) "John.6.42"
∷ word (ἡ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.6.42"
∷ word (ο ∷ ἴ ∷ δ ∷ α ∷ μ ∷ ε ∷ ν ∷ []) "John.6.42"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.6.42"
∷ word (π ∷ α ∷ τ ∷ έ ∷ ρ ∷ α ∷ []) "John.6.42"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.6.42"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.6.42"
∷ word (μ ∷ η ∷ τ ∷ έ ∷ ρ ∷ α ∷ []) "John.6.42"
∷ word (π ∷ ῶ ∷ ς ∷ []) "John.6.42"
∷ word (ν ∷ ῦ ∷ ν ∷ []) "John.6.42"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.6.42"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.6.42"
∷ word (Ἐ ∷ κ ∷ []) "John.6.42"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.6.42"
∷ word (ο ∷ ὐ ∷ ρ ∷ α ∷ ν ∷ ο ∷ ῦ ∷ []) "John.6.42"
∷ word (κ ∷ α ∷ τ ∷ α ∷ β ∷ έ ∷ β ∷ η ∷ κ ∷ α ∷ []) "John.6.42"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.6.43"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.6.43"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.6.43"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.6.43"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.6.43"
∷ word (Μ ∷ ὴ ∷ []) "John.6.43"
∷ word (γ ∷ ο ∷ γ ∷ γ ∷ ύ ∷ ζ ∷ ε ∷ τ ∷ ε ∷ []) "John.6.43"
∷ word (μ ∷ ε ∷ τ ∷ []) "John.6.43"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ή ∷ ∙λ ∷ ω ∷ ν ∷ []) "John.6.43"
∷ word (ο ∷ ὐ ∷ δ ∷ ε ∷ ὶ ∷ ς ∷ []) "John.6.44"
∷ word (δ ∷ ύ ∷ ν ∷ α ∷ τ ∷ α ∷ ι ∷ []) "John.6.44"
∷ word (ἐ ∷ ∙λ ∷ θ ∷ ε ∷ ῖ ∷ ν ∷ []) "John.6.44"
∷ word (π ∷ ρ ∷ ό ∷ ς ∷ []) "John.6.44"
∷ word (μ ∷ ε ∷ []) "John.6.44"
∷ word (ἐ ∷ ὰ ∷ ν ∷ []) "John.6.44"
∷ word (μ ∷ ὴ ∷ []) "John.6.44"
∷ word (ὁ ∷ []) "John.6.44"
∷ word (π ∷ α ∷ τ ∷ ὴ ∷ ρ ∷ []) "John.6.44"
∷ word (ὁ ∷ []) "John.6.44"
∷ word (π ∷ έ ∷ μ ∷ ψ ∷ α ∷ ς ∷ []) "John.6.44"
∷ word (μ ∷ ε ∷ []) "John.6.44"
∷ word (ἑ ∷ ∙λ ∷ κ ∷ ύ ∷ σ ∷ ῃ ∷ []) "John.6.44"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.6.44"
∷ word (κ ∷ ἀ ∷ γ ∷ ὼ ∷ []) "John.6.44"
∷ word (ἀ ∷ ν ∷ α ∷ σ ∷ τ ∷ ή ∷ σ ∷ ω ∷ []) "John.6.44"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.6.44"
∷ word (ἐ ∷ ν ∷ []) "John.6.44"
∷ word (τ ∷ ῇ ∷ []) "John.6.44"
∷ word (ἐ ∷ σ ∷ χ ∷ ά ∷ τ ∷ ῃ ∷ []) "John.6.44"
∷ word (ἡ ∷ μ ∷ έ ∷ ρ ∷ ᾳ ∷ []) "John.6.44"
∷ word (ἔ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.6.45"
∷ word (γ ∷ ε ∷ γ ∷ ρ ∷ α ∷ μ ∷ μ ∷ έ ∷ ν ∷ ο ∷ ν ∷ []) "John.6.45"
∷ word (ἐ ∷ ν ∷ []) "John.6.45"
∷ word (τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.6.45"
∷ word (π ∷ ρ ∷ ο ∷ φ ∷ ή ∷ τ ∷ α ∷ ι ∷ ς ∷ []) "John.6.45"
∷ word (Κ ∷ α ∷ ὶ ∷ []) "John.6.45"
∷ word (ἔ ∷ σ ∷ ο ∷ ν ∷ τ ∷ α ∷ ι ∷ []) "John.6.45"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.6.45"
∷ word (δ ∷ ι ∷ δ ∷ α ∷ κ ∷ τ ∷ ο ∷ ὶ ∷ []) "John.6.45"
∷ word (θ ∷ ε ∷ ο ∷ ῦ ∷ []) "John.6.45"
∷ word (π ∷ ᾶ ∷ ς ∷ []) "John.6.45"
∷ word (ὁ ∷ []) "John.6.45"
∷ word (ἀ ∷ κ ∷ ο ∷ ύ ∷ σ ∷ α ∷ ς ∷ []) "John.6.45"
∷ word (π ∷ α ∷ ρ ∷ ὰ ∷ []) "John.6.45"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.6.45"
∷ word (π ∷ α ∷ τ ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.6.45"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.6.45"
∷ word (μ ∷ α ∷ θ ∷ ὼ ∷ ν ∷ []) "John.6.45"
∷ word (ἔ ∷ ρ ∷ χ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.6.45"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.6.45"
∷ word (ἐ ∷ μ ∷ έ ∷ []) "John.6.45"
∷ word (ο ∷ ὐ ∷ χ ∷ []) "John.6.46"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.6.46"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.6.46"
∷ word (π ∷ α ∷ τ ∷ έ ∷ ρ ∷ α ∷ []) "John.6.46"
∷ word (ἑ ∷ ώ ∷ ρ ∷ α ∷ κ ∷ έ ∷ ν ∷ []) "John.6.46"
∷ word (τ ∷ ι ∷ ς ∷ []) "John.6.46"
∷ word (ε ∷ ἰ ∷ []) "John.6.46"
∷ word (μ ∷ ὴ ∷ []) "John.6.46"
∷ word (ὁ ∷ []) "John.6.46"
∷ word (ὢ ∷ ν ∷ []) "John.6.46"
∷ word (π ∷ α ∷ ρ ∷ ὰ ∷ []) "John.6.46"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.6.46"
∷ word (θ ∷ ε ∷ ο ∷ ῦ ∷ []) "John.6.46"
∷ word (ο ∷ ὗ ∷ τ ∷ ο ∷ ς ∷ []) "John.6.46"
∷ word (ἑ ∷ ώ ∷ ρ ∷ α ∷ κ ∷ ε ∷ ν ∷ []) "John.6.46"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.6.46"
∷ word (π ∷ α ∷ τ ∷ έ ∷ ρ ∷ α ∷ []) "John.6.46"
∷ word (ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.6.47"
∷ word (ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.6.47"
∷ word (∙λ ∷ έ ∷ γ ∷ ω ∷ []) "John.6.47"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.6.47"
∷ word (ὁ ∷ []) "John.6.47"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ ω ∷ ν ∷ []) "John.6.47"
∷ word (ἔ ∷ χ ∷ ε ∷ ι ∷ []) "John.6.47"
∷ word (ζ ∷ ω ∷ ὴ ∷ ν ∷ []) "John.6.47"
∷ word (α ∷ ἰ ∷ ώ ∷ ν ∷ ι ∷ ο ∷ ν ∷ []) "John.6.47"
∷ word (ἐ ∷ γ ∷ ώ ∷ []) "John.6.48"
∷ word (ε ∷ ἰ ∷ μ ∷ ι ∷ []) "John.6.48"
∷ word (ὁ ∷ []) "John.6.48"
∷ word (ἄ ∷ ρ ∷ τ ∷ ο ∷ ς ∷ []) "John.6.48"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.6.48"
∷ word (ζ ∷ ω ∷ ῆ ∷ ς ∷ []) "John.6.48"
∷ word (ο ∷ ἱ ∷ []) "John.6.49"
∷ word (π ∷ α ∷ τ ∷ έ ∷ ρ ∷ ε ∷ ς ∷ []) "John.6.49"
∷ word (ὑ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.6.49"
∷ word (ἔ ∷ φ ∷ α ∷ γ ∷ ο ∷ ν ∷ []) "John.6.49"
∷ word (ἐ ∷ ν ∷ []) "John.6.49"
∷ word (τ ∷ ῇ ∷ []) "John.6.49"
∷ word (ἐ ∷ ρ ∷ ή ∷ μ ∷ ῳ ∷ []) "John.6.49"
∷ word (τ ∷ ὸ ∷ []) "John.6.49"
∷ word (μ ∷ ά ∷ ν ∷ ν ∷ α ∷ []) "John.6.49"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.6.49"
∷ word (ἀ ∷ π ∷ έ ∷ θ ∷ α ∷ ν ∷ ο ∷ ν ∷ []) "John.6.49"
∷ word (ο ∷ ὗ ∷ τ ∷ ό ∷ ς ∷ []) "John.6.50"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.6.50"
∷ word (ὁ ∷ []) "John.6.50"
∷ word (ἄ ∷ ρ ∷ τ ∷ ο ∷ ς ∷ []) "John.6.50"
∷ word (ὁ ∷ []) "John.6.50"
∷ word (ἐ ∷ κ ∷ []) "John.6.50"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.6.50"
∷ word (ο ∷ ὐ ∷ ρ ∷ α ∷ ν ∷ ο ∷ ῦ ∷ []) "John.6.50"
∷ word (κ ∷ α ∷ τ ∷ α ∷ β ∷ α ∷ ί ∷ ν ∷ ω ∷ ν ∷ []) "John.6.50"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.6.50"
∷ word (τ ∷ ι ∷ ς ∷ []) "John.6.50"
∷ word (ἐ ∷ ξ ∷ []) "John.6.50"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.6.50"
∷ word (φ ∷ ά ∷ γ ∷ ῃ ∷ []) "John.6.50"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.6.50"
∷ word (μ ∷ ὴ ∷ []) "John.6.50"
∷ word (ἀ ∷ π ∷ ο ∷ θ ∷ ά ∷ ν ∷ ῃ ∷ []) "John.6.50"
∷ word (ἐ ∷ γ ∷ ώ ∷ []) "John.6.51"
∷ word (ε ∷ ἰ ∷ μ ∷ ι ∷ []) "John.6.51"
∷ word (ὁ ∷ []) "John.6.51"
∷ word (ἄ ∷ ρ ∷ τ ∷ ο ∷ ς ∷ []) "John.6.51"
∷ word (ὁ ∷ []) "John.6.51"
∷ word (ζ ∷ ῶ ∷ ν ∷ []) "John.6.51"
∷ word (ὁ ∷ []) "John.6.51"
∷ word (ἐ ∷ κ ∷ []) "John.6.51"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.6.51"
∷ word (ο ∷ ὐ ∷ ρ ∷ α ∷ ν ∷ ο ∷ ῦ ∷ []) "John.6.51"
∷ word (κ ∷ α ∷ τ ∷ α ∷ β ∷ ά ∷ ς ∷ []) "John.6.51"
∷ word (ἐ ∷ ά ∷ ν ∷ []) "John.6.51"
∷ word (τ ∷ ι ∷ ς ∷ []) "John.6.51"
∷ word (φ ∷ ά ∷ γ ∷ ῃ ∷ []) "John.6.51"
∷ word (ἐ ∷ κ ∷ []) "John.6.51"
∷ word (τ ∷ ο ∷ ύ ∷ τ ∷ ο ∷ υ ∷ []) "John.6.51"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.6.51"
∷ word (ἄ ∷ ρ ∷ τ ∷ ο ∷ υ ∷ []) "John.6.51"
∷ word (ζ ∷ ή ∷ σ ∷ ε ∷ ι ∷ []) "John.6.51"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.6.51"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.6.51"
∷ word (α ∷ ἰ ∷ ῶ ∷ ν ∷ α ∷ []) "John.6.51"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.6.51"
∷ word (ὁ ∷ []) "John.6.51"
∷ word (ἄ ∷ ρ ∷ τ ∷ ο ∷ ς ∷ []) "John.6.51"
∷ word (δ ∷ ὲ ∷ []) "John.6.51"
∷ word (ὃ ∷ ν ∷ []) "John.6.51"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.6.51"
∷ word (δ ∷ ώ ∷ σ ∷ ω ∷ []) "John.6.51"
∷ word (ἡ ∷ []) "John.6.51"
∷ word (σ ∷ ά ∷ ρ ∷ ξ ∷ []) "John.6.51"
∷ word (μ ∷ ο ∷ ύ ∷ []) "John.6.51"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.6.51"
∷ word (ὑ ∷ π ∷ ὲ ∷ ρ ∷ []) "John.6.51"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.6.51"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.6.51"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ υ ∷ []) "John.6.51"
∷ word (ζ ∷ ω ∷ ῆ ∷ ς ∷ []) "John.6.51"
∷ word (Ἐ ∷ μ ∷ ά ∷ χ ∷ ο ∷ ν ∷ τ ∷ ο ∷ []) "John.6.52"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.6.52"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.6.52"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ή ∷ ∙λ ∷ ο ∷ υ ∷ ς ∷ []) "John.6.52"
∷ word (ο ∷ ἱ ∷ []) "John.6.52"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ῖ ∷ ο ∷ ι ∷ []) "John.6.52"
∷ word (∙λ ∷ έ ∷ γ ∷ ο ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.6.52"
∷ word (Π ∷ ῶ ∷ ς ∷ []) "John.6.52"
∷ word (δ ∷ ύ ∷ ν ∷ α ∷ τ ∷ α ∷ ι ∷ []) "John.6.52"
∷ word (ο ∷ ὗ ∷ τ ∷ ο ∷ ς ∷ []) "John.6.52"
∷ word (ἡ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.6.52"
∷ word (δ ∷ ο ∷ ῦ ∷ ν ∷ α ∷ ι ∷ []) "John.6.52"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.6.52"
∷ word (σ ∷ ά ∷ ρ ∷ κ ∷ α ∷ []) "John.6.52"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.6.52"
∷ word (φ ∷ α ∷ γ ∷ ε ∷ ῖ ∷ ν ∷ []) "John.6.52"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.6.53"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.6.53"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.6.53"
∷ word (ὁ ∷ []) "John.6.53"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.6.53"
∷ word (Ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.6.53"
∷ word (ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.6.53"
∷ word (∙λ ∷ έ ∷ γ ∷ ω ∷ []) "John.6.53"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.6.53"
∷ word (ἐ ∷ ὰ ∷ ν ∷ []) "John.6.53"
∷ word (μ ∷ ὴ ∷ []) "John.6.53"
∷ word (φ ∷ ά ∷ γ ∷ η ∷ τ ∷ ε ∷ []) "John.6.53"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.6.53"
∷ word (σ ∷ ά ∷ ρ ∷ κ ∷ α ∷ []) "John.6.53"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.6.53"
∷ word (υ ∷ ἱ ∷ ο ∷ ῦ ∷ []) "John.6.53"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.6.53"
∷ word (ἀ ∷ ν ∷ θ ∷ ρ ∷ ώ ∷ π ∷ ο ∷ υ ∷ []) "John.6.53"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.6.53"
∷ word (π ∷ ί ∷ η ∷ τ ∷ ε ∷ []) "John.6.53"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.6.53"
∷ word (τ ∷ ὸ ∷ []) "John.6.53"
∷ word (α ∷ ἷ ∷ μ ∷ α ∷ []) "John.6.53"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.6.53"
∷ word (ἔ ∷ χ ∷ ε ∷ τ ∷ ε ∷ []) "John.6.53"
∷ word (ζ ∷ ω ∷ ὴ ∷ ν ∷ []) "John.6.53"
∷ word (ἐ ∷ ν ∷ []) "John.6.53"
∷ word (ἑ ∷ α ∷ υ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.6.53"
∷ word (ὁ ∷ []) "John.6.54"
∷ word (τ ∷ ρ ∷ ώ ∷ γ ∷ ω ∷ ν ∷ []) "John.6.54"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.6.54"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.6.54"
∷ word (σ ∷ ά ∷ ρ ∷ κ ∷ α ∷ []) "John.6.54"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.6.54"
∷ word (π ∷ ί ∷ ν ∷ ω ∷ ν ∷ []) "John.6.54"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.6.54"
∷ word (τ ∷ ὸ ∷ []) "John.6.54"
∷ word (α ∷ ἷ ∷ μ ∷ α ∷ []) "John.6.54"
∷ word (ἔ ∷ χ ∷ ε ∷ ι ∷ []) "John.6.54"
∷ word (ζ ∷ ω ∷ ὴ ∷ ν ∷ []) "John.6.54"
∷ word (α ∷ ἰ ∷ ώ ∷ ν ∷ ι ∷ ο ∷ ν ∷ []) "John.6.54"
∷ word (κ ∷ ἀ ∷ γ ∷ ὼ ∷ []) "John.6.54"
∷ word (ἀ ∷ ν ∷ α ∷ σ ∷ τ ∷ ή ∷ σ ∷ ω ∷ []) "John.6.54"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.6.54"
∷ word (τ ∷ ῇ ∷ []) "John.6.54"
∷ word (ἐ ∷ σ ∷ χ ∷ ά ∷ τ ∷ ῃ ∷ []) "John.6.54"
∷ word (ἡ ∷ μ ∷ έ ∷ ρ ∷ ᾳ ∷ []) "John.6.54"
∷ word (ἡ ∷ []) "John.6.55"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.6.55"
∷ word (σ ∷ ά ∷ ρ ∷ ξ ∷ []) "John.6.55"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.6.55"
∷ word (ἀ ∷ ∙λ ∷ η ∷ θ ∷ ή ∷ ς ∷ []) "John.6.55"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ []) "John.6.55"
∷ word (β ∷ ρ ∷ ῶ ∷ σ ∷ ι ∷ ς ∷ []) "John.6.55"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.6.55"
∷ word (τ ∷ ὸ ∷ []) "John.6.55"
∷ word (α ∷ ἷ ∷ μ ∷ ά ∷ []) "John.6.55"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.6.55"
∷ word (ἀ ∷ ∙λ ∷ η ∷ θ ∷ ή ∷ ς ∷ []) "John.6.55"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ []) "John.6.55"
∷ word (π ∷ ό ∷ σ ∷ ι ∷ ς ∷ []) "John.6.55"
∷ word (ὁ ∷ []) "John.6.56"
∷ word (τ ∷ ρ ∷ ώ ∷ γ ∷ ω ∷ ν ∷ []) "John.6.56"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.6.56"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.6.56"
∷ word (σ ∷ ά ∷ ρ ∷ κ ∷ α ∷ []) "John.6.56"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.6.56"
∷ word (π ∷ ί ∷ ν ∷ ω ∷ ν ∷ []) "John.6.56"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.6.56"
∷ word (τ ∷ ὸ ∷ []) "John.6.56"
∷ word (α ∷ ἷ ∷ μ ∷ α ∷ []) "John.6.56"
∷ word (ἐ ∷ ν ∷ []) "John.6.56"
∷ word (ἐ ∷ μ ∷ ο ∷ ὶ ∷ []) "John.6.56"
∷ word (μ ∷ έ ∷ ν ∷ ε ∷ ι ∷ []) "John.6.56"
∷ word (κ ∷ ἀ ∷ γ ∷ ὼ ∷ []) "John.6.56"
∷ word (ἐ ∷ ν ∷ []) "John.6.56"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.6.56"
∷ word (κ ∷ α ∷ θ ∷ ὼ ∷ ς ∷ []) "John.6.57"
∷ word (ἀ ∷ π ∷ έ ∷ σ ∷ τ ∷ ε ∷ ι ∷ ∙λ ∷ έ ∷ ν ∷ []) "John.6.57"
∷ word (μ ∷ ε ∷ []) "John.6.57"
∷ word (ὁ ∷ []) "John.6.57"
∷ word (ζ ∷ ῶ ∷ ν ∷ []) "John.6.57"
∷ word (π ∷ α ∷ τ ∷ ὴ ∷ ρ ∷ []) "John.6.57"
∷ word (κ ∷ ἀ ∷ γ ∷ ὼ ∷ []) "John.6.57"
∷ word (ζ ∷ ῶ ∷ []) "John.6.57"
∷ word (δ ∷ ι ∷ ὰ ∷ []) "John.6.57"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.6.57"
∷ word (π ∷ α ∷ τ ∷ έ ∷ ρ ∷ α ∷ []) "John.6.57"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.6.57"
∷ word (ὁ ∷ []) "John.6.57"
∷ word (τ ∷ ρ ∷ ώ ∷ γ ∷ ω ∷ ν ∷ []) "John.6.57"
∷ word (μ ∷ ε ∷ []) "John.6.57"
∷ word (κ ∷ ἀ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ο ∷ ς ∷ []) "John.6.57"
∷ word (ζ ∷ ή ∷ σ ∷ ε ∷ ι ∷ []) "John.6.57"
∷ word (δ ∷ ι ∷ []) "John.6.57"
∷ word (ἐ ∷ μ ∷ έ ∷ []) "John.6.57"
∷ word (ο ∷ ὗ ∷ τ ∷ ό ∷ ς ∷ []) "John.6.58"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.6.58"
∷ word (ὁ ∷ []) "John.6.58"
∷ word (ἄ ∷ ρ ∷ τ ∷ ο ∷ ς ∷ []) "John.6.58"
∷ word (ὁ ∷ []) "John.6.58"
∷ word (ἐ ∷ ξ ∷ []) "John.6.58"
∷ word (ο ∷ ὐ ∷ ρ ∷ α ∷ ν ∷ ο ∷ ῦ ∷ []) "John.6.58"
∷ word (κ ∷ α ∷ τ ∷ α ∷ β ∷ ά ∷ ς ∷ []) "John.6.58"
∷ word (ο ∷ ὐ ∷ []) "John.6.58"
∷ word (κ ∷ α ∷ θ ∷ ὼ ∷ ς ∷ []) "John.6.58"
∷ word (ἔ ∷ φ ∷ α ∷ γ ∷ ο ∷ ν ∷ []) "John.6.58"
∷ word (ο ∷ ἱ ∷ []) "John.6.58"
∷ word (π ∷ α ∷ τ ∷ έ ∷ ρ ∷ ε ∷ ς ∷ []) "John.6.58"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.6.58"
∷ word (ἀ ∷ π ∷ έ ∷ θ ∷ α ∷ ν ∷ ο ∷ ν ∷ []) "John.6.58"
∷ word (ὁ ∷ []) "John.6.58"
∷ word (τ ∷ ρ ∷ ώ ∷ γ ∷ ω ∷ ν ∷ []) "John.6.58"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ ν ∷ []) "John.6.58"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.6.58"
∷ word (ἄ ∷ ρ ∷ τ ∷ ο ∷ ν ∷ []) "John.6.58"
∷ word (ζ ∷ ή ∷ σ ∷ ε ∷ ι ∷ []) "John.6.58"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.6.58"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.6.58"
∷ word (α ∷ ἰ ∷ ῶ ∷ ν ∷ α ∷ []) "John.6.58"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.6.59"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.6.59"
∷ word (ἐ ∷ ν ∷ []) "John.6.59"
∷ word (σ ∷ υ ∷ ν ∷ α ∷ γ ∷ ω ∷ γ ∷ ῇ ∷ []) "John.6.59"
∷ word (δ ∷ ι ∷ δ ∷ ά ∷ σ ∷ κ ∷ ω ∷ ν ∷ []) "John.6.59"
∷ word (ἐ ∷ ν ∷ []) "John.6.59"
∷ word (Κ ∷ α ∷ φ ∷ α ∷ ρ ∷ ν ∷ α ∷ ο ∷ ύ ∷ μ ∷ []) "John.6.59"
∷ word (Π ∷ ο ∷ ∙λ ∷ ∙λ ∷ ο ∷ ὶ ∷ []) "John.6.60"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.6.60"
∷ word (ἀ ∷ κ ∷ ο ∷ ύ ∷ σ ∷ α ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.6.60"
∷ word (ἐ ∷ κ ∷ []) "John.6.60"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.6.60"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ ῶ ∷ ν ∷ []) "John.6.60"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.6.60"
∷ word (ε ∷ ἶ ∷ π ∷ α ∷ ν ∷ []) "John.6.60"
∷ word (Σ ∷ κ ∷ ∙λ ∷ η ∷ ρ ∷ ό ∷ ς ∷ []) "John.6.60"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.6.60"
∷ word (ὁ ∷ []) "John.6.60"
∷ word (∙λ ∷ ό ∷ γ ∷ ο ∷ ς ∷ []) "John.6.60"
∷ word (ο ∷ ὗ ∷ τ ∷ ο ∷ ς ∷ []) "John.6.60"
∷ word (τ ∷ ί ∷ ς ∷ []) "John.6.60"
∷ word (δ ∷ ύ ∷ ν ∷ α ∷ τ ∷ α ∷ ι ∷ []) "John.6.60"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.6.60"
∷ word (ἀ ∷ κ ∷ ο ∷ ύ ∷ ε ∷ ι ∷ ν ∷ []) "John.6.60"
∷ word (ε ∷ ἰ ∷ δ ∷ ὼ ∷ ς ∷ []) "John.6.61"
∷ word (δ ∷ ὲ ∷ []) "John.6.61"
∷ word (ὁ ∷ []) "John.6.61"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.6.61"
∷ word (ἐ ∷ ν ∷ []) "John.6.61"
∷ word (ἑ ∷ α ∷ υ ∷ τ ∷ ῷ ∷ []) "John.6.61"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.6.61"
∷ word (γ ∷ ο ∷ γ ∷ γ ∷ ύ ∷ ζ ∷ ο ∷ υ ∷ σ ∷ ι ∷ ν ∷ []) "John.6.61"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.6.61"
∷ word (τ ∷ ο ∷ ύ ∷ τ ∷ ο ∷ υ ∷ []) "John.6.61"
∷ word (ο ∷ ἱ ∷ []) "John.6.61"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ α ∷ ὶ ∷ []) "John.6.61"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.6.61"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.6.61"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.6.61"
∷ word (Τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.6.61"
∷ word (ὑ ∷ μ ∷ ᾶ ∷ ς ∷ []) "John.6.61"
∷ word (σ ∷ κ ∷ α ∷ ν ∷ δ ∷ α ∷ ∙λ ∷ ί ∷ ζ ∷ ε ∷ ι ∷ []) "John.6.61"
∷ word (ἐ ∷ ὰ ∷ ν ∷ []) "John.6.62"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.6.62"
∷ word (θ ∷ ε ∷ ω ∷ ρ ∷ ῆ ∷ τ ∷ ε ∷ []) "John.6.62"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.6.62"
∷ word (υ ∷ ἱ ∷ ὸ ∷ ν ∷ []) "John.6.62"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.6.62"
∷ word (ἀ ∷ ν ∷ θ ∷ ρ ∷ ώ ∷ π ∷ ο ∷ υ ∷ []) "John.6.62"
∷ word (ἀ ∷ ν ∷ α ∷ β ∷ α ∷ ί ∷ ν ∷ ο ∷ ν ∷ τ ∷ α ∷ []) "John.6.62"
∷ word (ὅ ∷ π ∷ ο ∷ υ ∷ []) "John.6.62"
∷ word (ἦ ∷ ν ∷ []) "John.6.62"
∷ word (τ ∷ ὸ ∷ []) "John.6.62"
∷ word (π ∷ ρ ∷ ό ∷ τ ∷ ε ∷ ρ ∷ ο ∷ ν ∷ []) "John.6.62"
∷ word (τ ∷ ὸ ∷ []) "John.6.63"
∷ word (π ∷ ν ∷ ε ∷ ῦ ∷ μ ∷ ά ∷ []) "John.6.63"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.6.63"
∷ word (τ ∷ ὸ ∷ []) "John.6.63"
∷ word (ζ ∷ ῳ ∷ ο ∷ π ∷ ο ∷ ι ∷ ο ∷ ῦ ∷ ν ∷ []) "John.6.63"
∷ word (ἡ ∷ []) "John.6.63"
∷ word (σ ∷ ὰ ∷ ρ ∷ ξ ∷ []) "John.6.63"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.6.63"
∷ word (ὠ ∷ φ ∷ ε ∷ ∙λ ∷ ε ∷ ῖ ∷ []) "John.6.63"
∷ word (ο ∷ ὐ ∷ δ ∷ έ ∷ ν ∷ []) "John.6.63"
∷ word (τ ∷ ὰ ∷ []) "John.6.63"
∷ word (ῥ ∷ ή ∷ μ ∷ α ∷ τ ∷ α ∷ []) "John.6.63"
∷ word (ἃ ∷ []) "John.6.63"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.6.63"
∷ word (∙λ ∷ ε ∷ ∙λ ∷ ά ∷ ∙λ ∷ η ∷ κ ∷ α ∷ []) "John.6.63"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.6.63"
∷ word (π ∷ ν ∷ ε ∷ ῦ ∷ μ ∷ ά ∷ []) "John.6.63"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.6.63"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.6.63"
∷ word (ζ ∷ ω ∷ ή ∷ []) "John.6.63"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.6.63"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.6.64"
∷ word (ε ∷ ἰ ∷ σ ∷ ὶ ∷ ν ∷ []) "John.6.64"
∷ word (ἐ ∷ ξ ∷ []) "John.6.64"
∷ word (ὑ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.6.64"
∷ word (τ ∷ ι ∷ ν ∷ ε ∷ ς ∷ []) "John.6.64"
∷ word (ο ∷ ἳ ∷ []) "John.6.64"
∷ word (ο ∷ ὐ ∷ []) "John.6.64"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ ο ∷ υ ∷ σ ∷ ι ∷ ν ∷ []) "John.6.64"
∷ word (ᾔ ∷ δ ∷ ε ∷ ι ∷ []) "John.6.64"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.6.64"
∷ word (ἐ ∷ ξ ∷ []) "John.6.64"
∷ word (ἀ ∷ ρ ∷ χ ∷ ῆ ∷ ς ∷ []) "John.6.64"
∷ word (ὁ ∷ []) "John.6.64"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.6.64"
∷ word (τ ∷ ί ∷ ν ∷ ε ∷ ς ∷ []) "John.6.64"
∷ word (ε ∷ ἰ ∷ σ ∷ ὶ ∷ ν ∷ []) "John.6.64"
∷ word (ο ∷ ἱ ∷ []) "John.6.64"
∷ word (μ ∷ ὴ ∷ []) "John.6.64"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ ο ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.6.64"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.6.64"
∷ word (τ ∷ ί ∷ ς ∷ []) "John.6.64"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.6.64"
∷ word (ὁ ∷ []) "John.6.64"
∷ word (π ∷ α ∷ ρ ∷ α ∷ δ ∷ ώ ∷ σ ∷ ω ∷ ν ∷ []) "John.6.64"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.6.64"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.6.65"
∷ word (ἔ ∷ ∙λ ∷ ε ∷ γ ∷ ε ∷ ν ∷ []) "John.6.65"
∷ word (Δ ∷ ι ∷ ὰ ∷ []) "John.6.65"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.6.65"
∷ word (ε ∷ ἴ ∷ ρ ∷ η ∷ κ ∷ α ∷ []) "John.6.65"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.6.65"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.6.65"
∷ word (ο ∷ ὐ ∷ δ ∷ ε ∷ ὶ ∷ ς ∷ []) "John.6.65"
∷ word (δ ∷ ύ ∷ ν ∷ α ∷ τ ∷ α ∷ ι ∷ []) "John.6.65"
∷ word (ἐ ∷ ∙λ ∷ θ ∷ ε ∷ ῖ ∷ ν ∷ []) "John.6.65"
∷ word (π ∷ ρ ∷ ό ∷ ς ∷ []) "John.6.65"
∷ word (μ ∷ ε ∷ []) "John.6.65"
∷ word (ἐ ∷ ὰ ∷ ν ∷ []) "John.6.65"
∷ word (μ ∷ ὴ ∷ []) "John.6.65"
∷ word (ᾖ ∷ []) "John.6.65"
∷ word (δ ∷ ε ∷ δ ∷ ο ∷ μ ∷ έ ∷ ν ∷ ο ∷ ν ∷ []) "John.6.65"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.6.65"
∷ word (ἐ ∷ κ ∷ []) "John.6.65"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.6.65"
∷ word (π ∷ α ∷ τ ∷ ρ ∷ ό ∷ ς ∷ []) "John.6.65"
∷ word (Ἐ ∷ κ ∷ []) "John.6.66"
∷ word (τ ∷ ο ∷ ύ ∷ τ ∷ ο ∷ υ ∷ []) "John.6.66"
∷ word (π ∷ ο ∷ ∙λ ∷ ∙λ ∷ ο ∷ ὶ ∷ []) "John.6.66"
∷ word (ἐ ∷ κ ∷ []) "John.6.66"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.6.66"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ ῶ ∷ ν ∷ []) "John.6.66"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.6.66"
∷ word (ἀ ∷ π ∷ ῆ ∷ ∙λ ∷ θ ∷ ο ∷ ν ∷ []) "John.6.66"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.6.66"
∷ word (τ ∷ ὰ ∷ []) "John.6.66"
∷ word (ὀ ∷ π ∷ ί ∷ σ ∷ ω ∷ []) "John.6.66"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.6.66"
∷ word (ο ∷ ὐ ∷ κ ∷ έ ∷ τ ∷ ι ∷ []) "John.6.66"
∷ word (μ ∷ ε ∷ τ ∷ []) "John.6.66"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.6.66"
∷ word (π ∷ ε ∷ ρ ∷ ι ∷ ε ∷ π ∷ ά ∷ τ ∷ ο ∷ υ ∷ ν ∷ []) "John.6.66"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.6.67"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.6.67"
∷ word (ὁ ∷ []) "John.6.67"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.6.67"
∷ word (τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.6.67"
∷ word (δ ∷ ώ ∷ δ ∷ ε ∷ κ ∷ α ∷ []) "John.6.67"
∷ word (Μ ∷ ὴ ∷ []) "John.6.67"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.6.67"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.6.67"
∷ word (θ ∷ έ ∷ ∙λ ∷ ε ∷ τ ∷ ε ∷ []) "John.6.67"
∷ word (ὑ ∷ π ∷ ά ∷ γ ∷ ε ∷ ι ∷ ν ∷ []) "John.6.67"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.6.68"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.6.68"
∷ word (Σ ∷ ί ∷ μ ∷ ω ∷ ν ∷ []) "John.6.68"
∷ word (Π ∷ έ ∷ τ ∷ ρ ∷ ο ∷ ς ∷ []) "John.6.68"
∷ word (Κ ∷ ύ ∷ ρ ∷ ι ∷ ε ∷ []) "John.6.68"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.6.68"
∷ word (τ ∷ ί ∷ ν ∷ α ∷ []) "John.6.68"
∷ word (ἀ ∷ π ∷ ε ∷ ∙λ ∷ ε ∷ υ ∷ σ ∷ ό ∷ μ ∷ ε ∷ θ ∷ α ∷ []) "John.6.68"
∷ word (ῥ ∷ ή ∷ μ ∷ α ∷ τ ∷ α ∷ []) "John.6.68"
∷ word (ζ ∷ ω ∷ ῆ ∷ ς ∷ []) "John.6.68"
∷ word (α ∷ ἰ ∷ ω ∷ ν ∷ ί ∷ ο ∷ υ ∷ []) "John.6.68"
∷ word (ἔ ∷ χ ∷ ε ∷ ι ∷ ς ∷ []) "John.6.68"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.6.69"
∷ word (ἡ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.6.69"
∷ word (π ∷ ε ∷ π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ κ ∷ α ∷ μ ∷ ε ∷ ν ∷ []) "John.6.69"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.6.69"
∷ word (ἐ ∷ γ ∷ ν ∷ ώ ∷ κ ∷ α ∷ μ ∷ ε ∷ ν ∷ []) "John.6.69"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.6.69"
∷ word (σ ∷ ὺ ∷ []) "John.6.69"
∷ word (ε ∷ ἶ ∷ []) "John.6.69"
∷ word (ὁ ∷ []) "John.6.69"
∷ word (ἅ ∷ γ ∷ ι ∷ ο ∷ ς ∷ []) "John.6.69"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.6.69"
∷ word (θ ∷ ε ∷ ο ∷ ῦ ∷ []) "John.6.69"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.6.70"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.6.70"
∷ word (ὁ ∷ []) "John.6.70"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.6.70"
∷ word (Ο ∷ ὐ ∷ κ ∷ []) "John.6.70"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.6.70"
∷ word (ὑ ∷ μ ∷ ᾶ ∷ ς ∷ []) "John.6.70"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.6.70"
∷ word (δ ∷ ώ ∷ δ ∷ ε ∷ κ ∷ α ∷ []) "John.6.70"
∷ word (ἐ ∷ ξ ∷ ε ∷ ∙λ ∷ ε ∷ ξ ∷ ά ∷ μ ∷ η ∷ ν ∷ []) "John.6.70"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.6.70"
∷ word (ἐ ∷ ξ ∷ []) "John.6.70"
∷ word (ὑ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.6.70"
∷ word (ε ∷ ἷ ∷ ς ∷ []) "John.6.70"
∷ word (δ ∷ ι ∷ ά ∷ β ∷ ο ∷ ∙λ ∷ ό ∷ ς ∷ []) "John.6.70"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.6.70"
∷ word (ἔ ∷ ∙λ ∷ ε ∷ γ ∷ ε ∷ ν ∷ []) "John.6.71"
∷ word (δ ∷ ὲ ∷ []) "John.6.71"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.6.71"
∷ word (Ἰ ∷ ο ∷ ύ ∷ δ ∷ α ∷ ν ∷ []) "John.6.71"
∷ word (Σ ∷ ί ∷ μ ∷ ω ∷ ν ∷ ο ∷ ς ∷ []) "John.6.71"
∷ word (Ἰ ∷ σ ∷ κ ∷ α ∷ ρ ∷ ι ∷ ώ ∷ τ ∷ ο ∷ υ ∷ []) "John.6.71"
∷ word (ο ∷ ὗ ∷ τ ∷ ο ∷ ς ∷ []) "John.6.71"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.6.71"
∷ word (ἔ ∷ μ ∷ ε ∷ ∙λ ∷ ∙λ ∷ ε ∷ ν ∷ []) "John.6.71"
∷ word (π ∷ α ∷ ρ ∷ α ∷ δ ∷ ι ∷ δ ∷ ό ∷ ν ∷ α ∷ ι ∷ []) "John.6.71"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.6.71"
∷ word (ε ∷ ἷ ∷ ς ∷ []) "John.6.71"
∷ word (ἐ ∷ κ ∷ []) "John.6.71"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.6.71"
∷ word (δ ∷ ώ ∷ δ ∷ ε ∷ κ ∷ α ∷ []) "John.6.71"
∷ word (Κ ∷ α ∷ ὶ ∷ []) "John.7.1"
∷ word (μ ∷ ε ∷ τ ∷ ὰ ∷ []) "John.7.1"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.7.1"
∷ word (π ∷ ε ∷ ρ ∷ ι ∷ ε ∷ π ∷ ά ∷ τ ∷ ε ∷ ι ∷ []) "John.7.1"
∷ word (ὁ ∷ []) "John.7.1"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.7.1"
∷ word (ἐ ∷ ν ∷ []) "John.7.1"
∷ word (τ ∷ ῇ ∷ []) "John.7.1"
∷ word (Γ ∷ α ∷ ∙λ ∷ ι ∷ ∙λ ∷ α ∷ ί ∷ ᾳ ∷ []) "John.7.1"
∷ word (ο ∷ ὐ ∷ []) "John.7.1"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.7.1"
∷ word (ἤ ∷ θ ∷ ε ∷ ∙λ ∷ ε ∷ ν ∷ []) "John.7.1"
∷ word (ἐ ∷ ν ∷ []) "John.7.1"
∷ word (τ ∷ ῇ ∷ []) "John.7.1"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ί ∷ ᾳ ∷ []) "John.7.1"
∷ word (π ∷ ε ∷ ρ ∷ ι ∷ π ∷ α ∷ τ ∷ ε ∷ ῖ ∷ ν ∷ []) "John.7.1"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.7.1"
∷ word (ἐ ∷ ζ ∷ ή ∷ τ ∷ ο ∷ υ ∷ ν ∷ []) "John.7.1"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.7.1"
∷ word (ο ∷ ἱ ∷ []) "John.7.1"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ῖ ∷ ο ∷ ι ∷ []) "John.7.1"
∷ word (ἀ ∷ π ∷ ο ∷ κ ∷ τ ∷ ε ∷ ῖ ∷ ν ∷ α ∷ ι ∷ []) "John.7.1"
∷ word (ἦ ∷ ν ∷ []) "John.7.2"
∷ word (δ ∷ ὲ ∷ []) "John.7.2"
∷ word (ἐ ∷ γ ∷ γ ∷ ὺ ∷ ς ∷ []) "John.7.2"
∷ word (ἡ ∷ []) "John.7.2"
∷ word (ἑ ∷ ο ∷ ρ ∷ τ ∷ ὴ ∷ []) "John.7.2"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.7.2"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ί ∷ ω ∷ ν ∷ []) "John.7.2"
∷ word (ἡ ∷ []) "John.7.2"
∷ word (σ ∷ κ ∷ η ∷ ν ∷ ο ∷ π ∷ η ∷ γ ∷ ί ∷ α ∷ []) "John.7.2"
∷ word (ε ∷ ἶ ∷ π ∷ ο ∷ ν ∷ []) "John.7.3"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.7.3"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.7.3"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.7.3"
∷ word (ο ∷ ἱ ∷ []) "John.7.3"
∷ word (ἀ ∷ δ ∷ ε ∷ ∙λ ∷ φ ∷ ο ∷ ὶ ∷ []) "John.7.3"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.7.3"
∷ word (Μ ∷ ε ∷ τ ∷ ά ∷ β ∷ η ∷ θ ∷ ι ∷ []) "John.7.3"
∷ word (ἐ ∷ ν ∷ τ ∷ ε ∷ ῦ ∷ θ ∷ ε ∷ ν ∷ []) "John.7.3"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.7.3"
∷ word (ὕ ∷ π ∷ α ∷ γ ∷ ε ∷ []) "John.7.3"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.7.3"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.7.3"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ί ∷ α ∷ ν ∷ []) "John.7.3"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.7.3"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.7.3"
∷ word (ο ∷ ἱ ∷ []) "John.7.3"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ α ∷ ί ∷ []) "John.7.3"
∷ word (σ ∷ ο ∷ υ ∷ []) "John.7.3"
∷ word (θ ∷ ε ∷ ω ∷ ρ ∷ ή ∷ σ ∷ ο ∷ υ ∷ σ ∷ ι ∷ ν ∷ []) "John.7.3"
∷ word (σ ∷ ο ∷ ῦ ∷ []) "John.7.3"
∷ word (τ ∷ ὰ ∷ []) "John.7.3"
∷ word (ἔ ∷ ρ ∷ γ ∷ α ∷ []) "John.7.3"
∷ word (ἃ ∷ []) "John.7.3"
∷ word (π ∷ ο ∷ ι ∷ ε ∷ ῖ ∷ ς ∷ []) "John.7.3"
∷ word (ο ∷ ὐ ∷ δ ∷ ε ∷ ὶ ∷ ς ∷ []) "John.7.4"
∷ word (γ ∷ ά ∷ ρ ∷ []) "John.7.4"
∷ word (τ ∷ ι ∷ []) "John.7.4"
∷ word (ἐ ∷ ν ∷ []) "John.7.4"
∷ word (κ ∷ ρ ∷ υ ∷ π ∷ τ ∷ ῷ ∷ []) "John.7.4"
∷ word (π ∷ ο ∷ ι ∷ ε ∷ ῖ ∷ []) "John.7.4"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.7.4"
∷ word (ζ ∷ η ∷ τ ∷ ε ∷ ῖ ∷ []) "John.7.4"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ς ∷ []) "John.7.4"
∷ word (ἐ ∷ ν ∷ []) "John.7.4"
∷ word (π ∷ α ∷ ρ ∷ ρ ∷ η ∷ σ ∷ ί ∷ ᾳ ∷ []) "John.7.4"
∷ word (ε ∷ ἶ ∷ ν ∷ α ∷ ι ∷ []) "John.7.4"
∷ word (ε ∷ ἰ ∷ []) "John.7.4"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.7.4"
∷ word (π ∷ ο ∷ ι ∷ ε ∷ ῖ ∷ ς ∷ []) "John.7.4"
∷ word (φ ∷ α ∷ ν ∷ έ ∷ ρ ∷ ω ∷ σ ∷ ο ∷ ν ∷ []) "John.7.4"
∷ word (σ ∷ ε ∷ α ∷ υ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.7.4"
∷ word (τ ∷ ῷ ∷ []) "John.7.4"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ῳ ∷ []) "John.7.4"
∷ word (ο ∷ ὐ ∷ δ ∷ ὲ ∷ []) "John.7.5"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.7.5"
∷ word (ο ∷ ἱ ∷ []) "John.7.5"
∷ word (ἀ ∷ δ ∷ ε ∷ ∙λ ∷ φ ∷ ο ∷ ὶ ∷ []) "John.7.5"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.7.5"
∷ word (ἐ ∷ π ∷ ί ∷ σ ∷ τ ∷ ε ∷ υ ∷ ο ∷ ν ∷ []) "John.7.5"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.7.5"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.7.5"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.7.6"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.7.6"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.7.6"
∷ word (ὁ ∷ []) "John.7.6"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.7.6"
∷ word (Ὁ ∷ []) "John.7.6"
∷ word (κ ∷ α ∷ ι ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.7.6"
∷ word (ὁ ∷ []) "John.7.6"
∷ word (ἐ ∷ μ ∷ ὸ ∷ ς ∷ []) "John.7.6"
∷ word (ο ∷ ὔ ∷ π ∷ ω ∷ []) "John.7.6"
∷ word (π ∷ ά ∷ ρ ∷ ε ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.7.6"
∷ word (ὁ ∷ []) "John.7.6"
∷ word (δ ∷ ὲ ∷ []) "John.7.6"
∷ word (κ ∷ α ∷ ι ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.7.6"
∷ word (ὁ ∷ []) "John.7.6"
∷ word (ὑ ∷ μ ∷ έ ∷ τ ∷ ε ∷ ρ ∷ ο ∷ ς ∷ []) "John.7.6"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ ο ∷ τ ∷ έ ∷ []) "John.7.6"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.7.6"
∷ word (ἕ ∷ τ ∷ ο ∷ ι ∷ μ ∷ ο ∷ ς ∷ []) "John.7.6"
∷ word (ο ∷ ὐ ∷ []) "John.7.7"
∷ word (δ ∷ ύ ∷ ν ∷ α ∷ τ ∷ α ∷ ι ∷ []) "John.7.7"
∷ word (ὁ ∷ []) "John.7.7"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ ς ∷ []) "John.7.7"
∷ word (μ ∷ ι ∷ σ ∷ ε ∷ ῖ ∷ ν ∷ []) "John.7.7"
∷ word (ὑ ∷ μ ∷ ᾶ ∷ ς ∷ []) "John.7.7"
∷ word (ἐ ∷ μ ∷ ὲ ∷ []) "John.7.7"
∷ word (δ ∷ ὲ ∷ []) "John.7.7"
∷ word (μ ∷ ι ∷ σ ∷ ε ∷ ῖ ∷ []) "John.7.7"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.7.7"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.7.7"
∷ word (μ ∷ α ∷ ρ ∷ τ ∷ υ ∷ ρ ∷ ῶ ∷ []) "John.7.7"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.7.7"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.7.7"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.7.7"
∷ word (τ ∷ ὰ ∷ []) "John.7.7"
∷ word (ἔ ∷ ρ ∷ γ ∷ α ∷ []) "John.7.7"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.7.7"
∷ word (π ∷ ο ∷ ν ∷ η ∷ ρ ∷ ά ∷ []) "John.7.7"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.7.7"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.7.8"
∷ word (ἀ ∷ ν ∷ ά ∷ β ∷ η ∷ τ ∷ ε ∷ []) "John.7.8"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.7.8"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.7.8"
∷ word (ἑ ∷ ο ∷ ρ ∷ τ ∷ ή ∷ ν ∷ []) "John.7.8"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.7.8"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.7.8"
∷ word (ἀ ∷ ν ∷ α ∷ β ∷ α ∷ ί ∷ ν ∷ ω ∷ []) "John.7.8"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.7.8"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.7.8"
∷ word (ἑ ∷ ο ∷ ρ ∷ τ ∷ ὴ ∷ ν ∷ []) "John.7.8"
∷ word (τ ∷ α ∷ ύ ∷ τ ∷ η ∷ ν ∷ []) "John.7.8"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.7.8"
∷ word (ὁ ∷ []) "John.7.8"
∷ word (ἐ ∷ μ ∷ ὸ ∷ ς ∷ []) "John.7.8"
∷ word (κ ∷ α ∷ ι ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.7.8"
∷ word (ο ∷ ὔ ∷ π ∷ ω ∷ []) "John.7.8"
∷ word (π ∷ ε ∷ π ∷ ∙λ ∷ ή ∷ ρ ∷ ω ∷ τ ∷ α ∷ ι ∷ []) "John.7.8"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.7.9"
∷ word (δ ∷ ὲ ∷ []) "John.7.9"
∷ word (ε ∷ ἰ ∷ π ∷ ὼ ∷ ν ∷ []) "John.7.9"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ς ∷ []) "John.7.9"
∷ word (ἔ ∷ μ ∷ ε ∷ ι ∷ ν ∷ ε ∷ ν ∷ []) "John.7.9"
∷ word (ἐ ∷ ν ∷ []) "John.7.9"
∷ word (τ ∷ ῇ ∷ []) "John.7.9"
∷ word (Γ ∷ α ∷ ∙λ ∷ ι ∷ ∙λ ∷ α ∷ ί ∷ ᾳ ∷ []) "John.7.9"
∷ word (Ὡ ∷ ς ∷ []) "John.7.10"
∷ word (δ ∷ ὲ ∷ []) "John.7.10"
∷ word (ἀ ∷ ν ∷ έ ∷ β ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.7.10"
∷ word (ο ∷ ἱ ∷ []) "John.7.10"
∷ word (ἀ ∷ δ ∷ ε ∷ ∙λ ∷ φ ∷ ο ∷ ὶ ∷ []) "John.7.10"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.7.10"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.7.10"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.7.10"
∷ word (ἑ ∷ ο ∷ ρ ∷ τ ∷ ή ∷ ν ∷ []) "John.7.10"
∷ word (τ ∷ ό ∷ τ ∷ ε ∷ []) "John.7.10"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.7.10"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ς ∷ []) "John.7.10"
∷ word (ἀ ∷ ν ∷ έ ∷ β ∷ η ∷ []) "John.7.10"
∷ word (ο ∷ ὐ ∷ []) "John.7.10"
∷ word (φ ∷ α ∷ ν ∷ ε ∷ ρ ∷ ῶ ∷ ς ∷ []) "John.7.10"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.7.10"
∷ word (ὡ ∷ ς ∷ []) "John.7.10"
∷ word (ἐ ∷ ν ∷ []) "John.7.10"
∷ word (κ ∷ ρ ∷ υ ∷ π ∷ τ ∷ ῷ ∷ []) "John.7.10"
∷ word (ο ∷ ἱ ∷ []) "John.7.11"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.7.11"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ῖ ∷ ο ∷ ι ∷ []) "John.7.11"
∷ word (ἐ ∷ ζ ∷ ή ∷ τ ∷ ο ∷ υ ∷ ν ∷ []) "John.7.11"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.7.11"
∷ word (ἐ ∷ ν ∷ []) "John.7.11"
∷ word (τ ∷ ῇ ∷ []) "John.7.11"
∷ word (ἑ ∷ ο ∷ ρ ∷ τ ∷ ῇ ∷ []) "John.7.11"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.7.11"
∷ word (ἔ ∷ ∙λ ∷ ε ∷ γ ∷ ο ∷ ν ∷ []) "John.7.11"
∷ word (Π ∷ ο ∷ ῦ ∷ []) "John.7.11"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.7.11"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ο ∷ ς ∷ []) "John.7.11"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.7.12"
∷ word (γ ∷ ο ∷ γ ∷ γ ∷ υ ∷ σ ∷ μ ∷ ὸ ∷ ς ∷ []) "John.7.12"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.7.12"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.7.12"
∷ word (ἦ ∷ ν ∷ []) "John.7.12"
∷ word (π ∷ ο ∷ ∙λ ∷ ὺ ∷ ς ∷ []) "John.7.12"
∷ word (ἐ ∷ ν ∷ []) "John.7.12"
∷ word (τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.7.12"
∷ word (ὄ ∷ χ ∷ ∙λ ∷ ο ∷ ι ∷ ς ∷ []) "John.7.12"
∷ word (ο ∷ ἱ ∷ []) "John.7.12"
∷ word (μ ∷ ὲ ∷ ν ∷ []) "John.7.12"
∷ word (ἔ ∷ ∙λ ∷ ε ∷ γ ∷ ο ∷ ν ∷ []) "John.7.12"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.7.12"
∷ word (Ἀ ∷ γ ∷ α ∷ θ ∷ ό ∷ ς ∷ []) "John.7.12"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.7.12"
∷ word (ἄ ∷ ∙λ ∷ ∙λ ∷ ο ∷ ι ∷ []) "John.7.12"
∷ word (δ ∷ ὲ ∷ []) "John.7.12"
∷ word (ἔ ∷ ∙λ ∷ ε ∷ γ ∷ ο ∷ ν ∷ []) "John.7.12"
∷ word (Ο ∷ ὔ ∷ []) "John.7.12"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.7.12"
∷ word (π ∷ ∙λ ∷ α ∷ ν ∷ ᾷ ∷ []) "John.7.12"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.7.12"
∷ word (ὄ ∷ χ ∷ ∙λ ∷ ο ∷ ν ∷ []) "John.7.12"
∷ word (ο ∷ ὐ ∷ δ ∷ ε ∷ ὶ ∷ ς ∷ []) "John.7.13"
∷ word (μ ∷ έ ∷ ν ∷ τ ∷ ο ∷ ι ∷ []) "John.7.13"
∷ word (π ∷ α ∷ ρ ∷ ρ ∷ η ∷ σ ∷ ί ∷ ᾳ ∷ []) "John.7.13"
∷ word (ἐ ∷ ∙λ ∷ ά ∷ ∙λ ∷ ε ∷ ι ∷ []) "John.7.13"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.7.13"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.7.13"
∷ word (δ ∷ ι ∷ ὰ ∷ []) "John.7.13"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.7.13"
∷ word (φ ∷ ό ∷ β ∷ ο ∷ ν ∷ []) "John.7.13"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.7.13"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ί ∷ ω ∷ ν ∷ []) "John.7.13"
∷ word (Ἤ ∷ δ ∷ η ∷ []) "John.7.14"
∷ word (δ ∷ ὲ ∷ []) "John.7.14"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.7.14"
∷ word (ἑ ∷ ο ∷ ρ ∷ τ ∷ ῆ ∷ ς ∷ []) "John.7.14"
∷ word (μ ∷ ε ∷ σ ∷ ο ∷ ύ ∷ σ ∷ η ∷ ς ∷ []) "John.7.14"
∷ word (ἀ ∷ ν ∷ έ ∷ β ∷ η ∷ []) "John.7.14"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.7.14"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.7.14"
∷ word (τ ∷ ὸ ∷ []) "John.7.14"
∷ word (ἱ ∷ ε ∷ ρ ∷ ὸ ∷ ν ∷ []) "John.7.14"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.7.14"
∷ word (ἐ ∷ δ ∷ ί ∷ δ ∷ α ∷ σ ∷ κ ∷ ε ∷ ν ∷ []) "John.7.14"
∷ word (ἐ ∷ θ ∷ α ∷ ύ ∷ μ ∷ α ∷ ζ ∷ ο ∷ ν ∷ []) "John.7.15"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.7.15"
∷ word (ο ∷ ἱ ∷ []) "John.7.15"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ῖ ∷ ο ∷ ι ∷ []) "John.7.15"
∷ word (∙λ ∷ έ ∷ γ ∷ ο ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.7.15"
∷ word (Π ∷ ῶ ∷ ς ∷ []) "John.7.15"
∷ word (ο ∷ ὗ ∷ τ ∷ ο ∷ ς ∷ []) "John.7.15"
∷ word (γ ∷ ρ ∷ ά ∷ μ ∷ μ ∷ α ∷ τ ∷ α ∷ []) "John.7.15"
∷ word (ο ∷ ἶ ∷ δ ∷ ε ∷ ν ∷ []) "John.7.15"
∷ word (μ ∷ ὴ ∷ []) "John.7.15"
∷ word (μ ∷ ε ∷ μ ∷ α ∷ θ ∷ η ∷ κ ∷ ώ ∷ ς ∷ []) "John.7.15"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.7.16"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.7.16"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.7.16"
∷ word (ὁ ∷ []) "John.7.16"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.7.16"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.7.16"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.7.16"
∷ word (Ἡ ∷ []) "John.7.16"
∷ word (ἐ ∷ μ ∷ ὴ ∷ []) "John.7.16"
∷ word (δ ∷ ι ∷ δ ∷ α ∷ χ ∷ ὴ ∷ []) "John.7.16"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.7.16"
∷ word (ἔ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.7.16"
∷ word (ἐ ∷ μ ∷ ὴ ∷ []) "John.7.16"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.7.16"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.7.16"
∷ word (π ∷ έ ∷ μ ∷ ψ ∷ α ∷ ν ∷ τ ∷ ό ∷ ς ∷ []) "John.7.16"
∷ word (μ ∷ ε ∷ []) "John.7.16"
∷ word (ἐ ∷ ά ∷ ν ∷ []) "John.7.17"
∷ word (τ ∷ ι ∷ ς ∷ []) "John.7.17"
∷ word (θ ∷ έ ∷ ∙λ ∷ ῃ ∷ []) "John.7.17"
∷ word (τ ∷ ὸ ∷ []) "John.7.17"
∷ word (θ ∷ έ ∷ ∙λ ∷ η ∷ μ ∷ α ∷ []) "John.7.17"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.7.17"
∷ word (π ∷ ο ∷ ι ∷ ε ∷ ῖ ∷ ν ∷ []) "John.7.17"
∷ word (γ ∷ ν ∷ ώ ∷ σ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.7.17"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.7.17"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.7.17"
∷ word (δ ∷ ι ∷ δ ∷ α ∷ χ ∷ ῆ ∷ ς ∷ []) "John.7.17"
∷ word (π ∷ ό ∷ τ ∷ ε ∷ ρ ∷ ο ∷ ν ∷ []) "John.7.17"
∷ word (ἐ ∷ κ ∷ []) "John.7.17"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.7.17"
∷ word (θ ∷ ε ∷ ο ∷ ῦ ∷ []) "John.7.17"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.7.17"
∷ word (ἢ ∷ []) "John.7.17"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.7.17"
∷ word (ἀ ∷ π ∷ []) "John.7.17"
∷ word (ἐ ∷ μ ∷ α ∷ υ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.7.17"
∷ word (∙λ ∷ α ∷ ∙λ ∷ ῶ ∷ []) "John.7.17"
∷ word (ὁ ∷ []) "John.7.18"
∷ word (ἀ ∷ φ ∷ []) "John.7.18"
∷ word (ἑ ∷ α ∷ υ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.7.18"
∷ word (∙λ ∷ α ∷ ∙λ ∷ ῶ ∷ ν ∷ []) "John.7.18"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.7.18"
∷ word (δ ∷ ό ∷ ξ ∷ α ∷ ν ∷ []) "John.7.18"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.7.18"
∷ word (ἰ ∷ δ ∷ ί ∷ α ∷ ν ∷ []) "John.7.18"
∷ word (ζ ∷ η ∷ τ ∷ ε ∷ ῖ ∷ []) "John.7.18"
∷ word (ὁ ∷ []) "John.7.18"
∷ word (δ ∷ ὲ ∷ []) "John.7.18"
∷ word (ζ ∷ η ∷ τ ∷ ῶ ∷ ν ∷ []) "John.7.18"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.7.18"
∷ word (δ ∷ ό ∷ ξ ∷ α ∷ ν ∷ []) "John.7.18"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.7.18"
∷ word (π ∷ έ ∷ μ ∷ ψ ∷ α ∷ ν ∷ τ ∷ ο ∷ ς ∷ []) "John.7.18"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.7.18"
∷ word (ο ∷ ὗ ∷ τ ∷ ο ∷ ς ∷ []) "John.7.18"
∷ word (ἀ ∷ ∙λ ∷ η ∷ θ ∷ ή ∷ ς ∷ []) "John.7.18"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.7.18"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.7.18"
∷ word (ἀ ∷ δ ∷ ι ∷ κ ∷ ί ∷ α ∷ []) "John.7.18"
∷ word (ἐ ∷ ν ∷ []) "John.7.18"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.7.18"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.7.18"
∷ word (ἔ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.7.18"
∷ word (Ο ∷ ὐ ∷ []) "John.7.19"
∷ word (Μ ∷ ω ∷ ϋ ∷ σ ∷ ῆ ∷ ς ∷ []) "John.7.19"
∷ word (δ ∷ έ ∷ δ ∷ ω ∷ κ ∷ ε ∷ ν ∷ []) "John.7.19"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.7.19"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.7.19"
∷ word (ν ∷ ό ∷ μ ∷ ο ∷ ν ∷ []) "John.7.19"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.7.19"
∷ word (ο ∷ ὐ ∷ δ ∷ ε ∷ ὶ ∷ ς ∷ []) "John.7.19"
∷ word (ἐ ∷ ξ ∷ []) "John.7.19"
∷ word (ὑ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.7.19"
∷ word (π ∷ ο ∷ ι ∷ ε ∷ ῖ ∷ []) "John.7.19"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.7.19"
∷ word (ν ∷ ό ∷ μ ∷ ο ∷ ν ∷ []) "John.7.19"
∷ word (τ ∷ ί ∷ []) "John.7.19"
∷ word (μ ∷ ε ∷ []) "John.7.19"
∷ word (ζ ∷ η ∷ τ ∷ ε ∷ ῖ ∷ τ ∷ ε ∷ []) "John.7.19"
∷ word (ἀ ∷ π ∷ ο ∷ κ ∷ τ ∷ ε ∷ ῖ ∷ ν ∷ α ∷ ι ∷ []) "John.7.19"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.7.20"
∷ word (ὁ ∷ []) "John.7.20"
∷ word (ὄ ∷ χ ∷ ∙λ ∷ ο ∷ ς ∷ []) "John.7.20"
∷ word (Δ ∷ α ∷ ι ∷ μ ∷ ό ∷ ν ∷ ι ∷ ο ∷ ν ∷ []) "John.7.20"
∷ word (ἔ ∷ χ ∷ ε ∷ ι ∷ ς ∷ []) "John.7.20"
∷ word (τ ∷ ί ∷ ς ∷ []) "John.7.20"
∷ word (σ ∷ ε ∷ []) "John.7.20"
∷ word (ζ ∷ η ∷ τ ∷ ε ∷ ῖ ∷ []) "John.7.20"
∷ word (ἀ ∷ π ∷ ο ∷ κ ∷ τ ∷ ε ∷ ῖ ∷ ν ∷ α ∷ ι ∷ []) "John.7.20"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.7.21"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.7.21"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.7.21"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.7.21"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.7.21"
∷ word (Ἓ ∷ ν ∷ []) "John.7.21"
∷ word (ἔ ∷ ρ ∷ γ ∷ ο ∷ ν ∷ []) "John.7.21"
∷ word (ἐ ∷ π ∷ ο ∷ ί ∷ η ∷ σ ∷ α ∷ []) "John.7.21"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.7.21"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.7.21"
∷ word (θ ∷ α ∷ υ ∷ μ ∷ ά ∷ ζ ∷ ε ∷ τ ∷ ε ∷ []) "John.7.21"
∷ word (δ ∷ ι ∷ ὰ ∷ []) "John.7.22"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.7.22"
∷ word (Μ ∷ ω ∷ ϋ ∷ σ ∷ ῆ ∷ ς ∷ []) "John.7.22"
∷ word (δ ∷ έ ∷ δ ∷ ω ∷ κ ∷ ε ∷ ν ∷ []) "John.7.22"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.7.22"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.7.22"
∷ word (π ∷ ε ∷ ρ ∷ ι ∷ τ ∷ ο ∷ μ ∷ ή ∷ ν ∷ []) "John.7.22"
∷ word (ο ∷ ὐ ∷ χ ∷ []) "John.7.22"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.7.22"
∷ word (ἐ ∷ κ ∷ []) "John.7.22"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.7.22"
∷ word (Μ ∷ ω ∷ ϋ ∷ σ ∷ έ ∷ ω ∷ ς ∷ []) "John.7.22"
∷ word (ἐ ∷ σ ∷ τ ∷ ὶ ∷ ν ∷ []) "John.7.22"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ []) "John.7.22"
∷ word (ἐ ∷ κ ∷ []) "John.7.22"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.7.22"
∷ word (π ∷ α ∷ τ ∷ έ ∷ ρ ∷ ω ∷ ν ∷ []) "John.7.22"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.7.22"
∷ word (ἐ ∷ ν ∷ []) "John.7.22"
∷ word (σ ∷ α ∷ β ∷ β ∷ ά ∷ τ ∷ ῳ ∷ []) "John.7.22"
∷ word (π ∷ ε ∷ ρ ∷ ι ∷ τ ∷ έ ∷ μ ∷ ν ∷ ε ∷ τ ∷ ε ∷ []) "John.7.22"
∷ word (ἄ ∷ ν ∷ θ ∷ ρ ∷ ω ∷ π ∷ ο ∷ ν ∷ []) "John.7.22"
∷ word (ε ∷ ἰ ∷ []) "John.7.23"
∷ word (π ∷ ε ∷ ρ ∷ ι ∷ τ ∷ ο ∷ μ ∷ ὴ ∷ ν ∷ []) "John.7.23"
∷ word (∙λ ∷ α ∷ μ ∷ β ∷ ά ∷ ν ∷ ε ∷ ι ∷ []) "John.7.23"
∷ word (ἄ ∷ ν ∷ θ ∷ ρ ∷ ω ∷ π ∷ ο ∷ ς ∷ []) "John.7.23"
∷ word (ἐ ∷ ν ∷ []) "John.7.23"
∷ word (σ ∷ α ∷ β ∷ β ∷ ά ∷ τ ∷ ῳ ∷ []) "John.7.23"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.7.23"
∷ word (μ ∷ ὴ ∷ []) "John.7.23"
∷ word (∙λ ∷ υ ∷ θ ∷ ῇ ∷ []) "John.7.23"
∷ word (ὁ ∷ []) "John.7.23"
∷ word (ν ∷ ό ∷ μ ∷ ο ∷ ς ∷ []) "John.7.23"
∷ word (Μ ∷ ω ∷ ϋ ∷ σ ∷ έ ∷ ω ∷ ς ∷ []) "John.7.23"
∷ word (ἐ ∷ μ ∷ ο ∷ ὶ ∷ []) "John.7.23"
∷ word (χ ∷ ο ∷ ∙λ ∷ ᾶ ∷ τ ∷ ε ∷ []) "John.7.23"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.7.23"
∷ word (ὅ ∷ ∙λ ∷ ο ∷ ν ∷ []) "John.7.23"
∷ word (ἄ ∷ ν ∷ θ ∷ ρ ∷ ω ∷ π ∷ ο ∷ ν ∷ []) "John.7.23"
∷ word (ὑ ∷ γ ∷ ι ∷ ῆ ∷ []) "John.7.23"
∷ word (ἐ ∷ π ∷ ο ∷ ί ∷ η ∷ σ ∷ α ∷ []) "John.7.23"
∷ word (ἐ ∷ ν ∷ []) "John.7.23"
∷ word (σ ∷ α ∷ β ∷ β ∷ ά ∷ τ ∷ ῳ ∷ []) "John.7.23"
∷ word (μ ∷ ὴ ∷ []) "John.7.24"
∷ word (κ ∷ ρ ∷ ί ∷ ν ∷ ε ∷ τ ∷ ε ∷ []) "John.7.24"
∷ word (κ ∷ α ∷ τ ∷ []) "John.7.24"
∷ word (ὄ ∷ ψ ∷ ι ∷ ν ∷ []) "John.7.24"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.7.24"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.7.24"
∷ word (δ ∷ ι ∷ κ ∷ α ∷ ί ∷ α ∷ ν ∷ []) "John.7.24"
∷ word (κ ∷ ρ ∷ ί ∷ σ ∷ ι ∷ ν ∷ []) "John.7.24"
∷ word (κ ∷ ρ ∷ ί ∷ ν ∷ ε ∷ τ ∷ ε ∷ []) "John.7.24"
∷ word (Ἔ ∷ ∙λ ∷ ε ∷ γ ∷ ο ∷ ν ∷ []) "John.7.25"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.7.25"
∷ word (τ ∷ ι ∷ ν ∷ ε ∷ ς ∷ []) "John.7.25"
∷ word (ἐ ∷ κ ∷ []) "John.7.25"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.7.25"
∷ word (Ἱ ∷ ε ∷ ρ ∷ ο ∷ σ ∷ ο ∷ ∙λ ∷ υ ∷ μ ∷ ι ∷ τ ∷ ῶ ∷ ν ∷ []) "John.7.25"
∷ word (Ο ∷ ὐ ∷ χ ∷ []) "John.7.25"
∷ word (ο ∷ ὗ ∷ τ ∷ ό ∷ ς ∷ []) "John.7.25"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.7.25"
∷ word (ὃ ∷ ν ∷ []) "John.7.25"
∷ word (ζ ∷ η ∷ τ ∷ ο ∷ ῦ ∷ σ ∷ ι ∷ ν ∷ []) "John.7.25"
∷ word (ἀ ∷ π ∷ ο ∷ κ ∷ τ ∷ ε ∷ ῖ ∷ ν ∷ α ∷ ι ∷ []) "John.7.25"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.7.26"
∷ word (ἴ ∷ δ ∷ ε ∷ []) "John.7.26"
∷ word (π ∷ α ∷ ρ ∷ ρ ∷ η ∷ σ ∷ ί ∷ ᾳ ∷ []) "John.7.26"
∷ word (∙λ ∷ α ∷ ∙λ ∷ ε ∷ ῖ ∷ []) "John.7.26"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.7.26"
∷ word (ο ∷ ὐ ∷ δ ∷ ὲ ∷ ν ∷ []) "John.7.26"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.7.26"
∷ word (∙λ ∷ έ ∷ γ ∷ ο ∷ υ ∷ σ ∷ ι ∷ ν ∷ []) "John.7.26"
∷ word (μ ∷ ή ∷ π ∷ ο ∷ τ ∷ ε ∷ []) "John.7.26"
∷ word (ἀ ∷ ∙λ ∷ η ∷ θ ∷ ῶ ∷ ς ∷ []) "John.7.26"
∷ word (ἔ ∷ γ ∷ ν ∷ ω ∷ σ ∷ α ∷ ν ∷ []) "John.7.26"
∷ word (ο ∷ ἱ ∷ []) "John.7.26"
∷ word (ἄ ∷ ρ ∷ χ ∷ ο ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.7.26"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.7.26"
∷ word (ο ∷ ὗ ∷ τ ∷ ό ∷ ς ∷ []) "John.7.26"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.7.26"
∷ word (ὁ ∷ []) "John.7.26"
∷ word (χ ∷ ρ ∷ ι ∷ σ ∷ τ ∷ ό ∷ ς ∷ []) "John.7.26"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.7.27"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ ν ∷ []) "John.7.27"
∷ word (ο ∷ ἴ ∷ δ ∷ α ∷ μ ∷ ε ∷ ν ∷ []) "John.7.27"
∷ word (π ∷ ό ∷ θ ∷ ε ∷ ν ∷ []) "John.7.27"
∷ word (ἐ ∷ σ ∷ τ ∷ ί ∷ ν ∷ []) "John.7.27"
∷ word (ὁ ∷ []) "John.7.27"
∷ word (δ ∷ ὲ ∷ []) "John.7.27"
∷ word (χ ∷ ρ ∷ ι ∷ σ ∷ τ ∷ ὸ ∷ ς ∷ []) "John.7.27"
∷ word (ὅ ∷ τ ∷ α ∷ ν ∷ []) "John.7.27"
∷ word (ἔ ∷ ρ ∷ χ ∷ η ∷ τ ∷ α ∷ ι ∷ []) "John.7.27"
∷ word (ο ∷ ὐ ∷ δ ∷ ε ∷ ὶ ∷ ς ∷ []) "John.7.27"
∷ word (γ ∷ ι ∷ ν ∷ ώ ∷ σ ∷ κ ∷ ε ∷ ι ∷ []) "John.7.27"
∷ word (π ∷ ό ∷ θ ∷ ε ∷ ν ∷ []) "John.7.27"
∷ word (ἐ ∷ σ ∷ τ ∷ ί ∷ ν ∷ []) "John.7.27"
∷ word (ἔ ∷ κ ∷ ρ ∷ α ∷ ξ ∷ ε ∷ ν ∷ []) "John.7.28"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.7.28"
∷ word (ἐ ∷ ν ∷ []) "John.7.28"
∷ word (τ ∷ ῷ ∷ []) "John.7.28"
∷ word (ἱ ∷ ε ∷ ρ ∷ ῷ ∷ []) "John.7.28"
∷ word (δ ∷ ι ∷ δ ∷ ά ∷ σ ∷ κ ∷ ω ∷ ν ∷ []) "John.7.28"
∷ word (ὁ ∷ []) "John.7.28"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.7.28"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.7.28"
∷ word (∙λ ∷ έ ∷ γ ∷ ω ∷ ν ∷ []) "John.7.28"
∷ word (Κ ∷ ἀ ∷ μ ∷ ὲ ∷ []) "John.7.28"
∷ word (ο ∷ ἴ ∷ δ ∷ α ∷ τ ∷ ε ∷ []) "John.7.28"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.7.28"
∷ word (ο ∷ ἴ ∷ δ ∷ α ∷ τ ∷ ε ∷ []) "John.7.28"
∷ word (π ∷ ό ∷ θ ∷ ε ∷ ν ∷ []) "John.7.28"
∷ word (ε ∷ ἰ ∷ μ ∷ ί ∷ []) "John.7.28"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.7.28"
∷ word (ἀ ∷ π ∷ []) "John.7.28"
∷ word (ἐ ∷ μ ∷ α ∷ υ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.7.28"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.7.28"
∷ word (ἐ ∷ ∙λ ∷ ή ∷ ∙λ ∷ υ ∷ θ ∷ α ∷ []) "John.7.28"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ []) "John.7.28"
∷ word (ἔ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.7.28"
∷ word (ἀ ∷ ∙λ ∷ η ∷ θ ∷ ι ∷ ν ∷ ὸ ∷ ς ∷ []) "John.7.28"
∷ word (ὁ ∷ []) "John.7.28"
∷ word (π ∷ έ ∷ μ ∷ ψ ∷ α ∷ ς ∷ []) "John.7.28"
∷ word (μ ∷ ε ∷ []) "John.7.28"
∷ word (ὃ ∷ ν ∷ []) "John.7.28"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.7.28"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.7.28"
∷ word (ο ∷ ἴ ∷ δ ∷ α ∷ τ ∷ ε ∷ []) "John.7.28"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.7.29"
∷ word (ο ∷ ἶ ∷ δ ∷ α ∷ []) "John.7.29"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.7.29"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.7.29"
∷ word (π ∷ α ∷ ρ ∷ []) "John.7.29"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.7.29"
∷ word (ε ∷ ἰ ∷ μ ∷ ι ∷ []) "John.7.29"
∷ word (κ ∷ ἀ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ό ∷ ς ∷ []) "John.7.29"
∷ word (μ ∷ ε ∷ []) "John.7.29"
∷ word (ἀ ∷ π ∷ έ ∷ σ ∷ τ ∷ ε ∷ ι ∷ ∙λ ∷ ε ∷ ν ∷ []) "John.7.29"
∷ word (ἐ ∷ ζ ∷ ή ∷ τ ∷ ο ∷ υ ∷ ν ∷ []) "John.7.30"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.7.30"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.7.30"
∷ word (π ∷ ι ∷ ά ∷ σ ∷ α ∷ ι ∷ []) "John.7.30"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.7.30"
∷ word (ο ∷ ὐ ∷ δ ∷ ε ∷ ὶ ∷ ς ∷ []) "John.7.30"
∷ word (ἐ ∷ π ∷ έ ∷ β ∷ α ∷ ∙λ ∷ ε ∷ ν ∷ []) "John.7.30"
∷ word (ἐ ∷ π ∷ []) "John.7.30"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.7.30"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.7.30"
∷ word (χ ∷ ε ∷ ῖ ∷ ρ ∷ α ∷ []) "John.7.30"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.7.30"
∷ word (ο ∷ ὔ ∷ π ∷ ω ∷ []) "John.7.30"
∷ word (ἐ ∷ ∙λ ∷ η ∷ ∙λ ∷ ύ ∷ θ ∷ ε ∷ ι ∷ []) "John.7.30"
∷ word (ἡ ∷ []) "John.7.30"
∷ word (ὥ ∷ ρ ∷ α ∷ []) "John.7.30"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.7.30"
∷ word (ἐ ∷ κ ∷ []) "John.7.31"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.7.31"
∷ word (ὄ ∷ χ ∷ ∙λ ∷ ο ∷ υ ∷ []) "John.7.31"
∷ word (δ ∷ ὲ ∷ []) "John.7.31"
∷ word (π ∷ ο ∷ ∙λ ∷ ∙λ ∷ ο ∷ ὶ ∷ []) "John.7.31"
∷ word (ἐ ∷ π ∷ ί ∷ σ ∷ τ ∷ ε ∷ υ ∷ σ ∷ α ∷ ν ∷ []) "John.7.31"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.7.31"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.7.31"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.7.31"
∷ word (ἔ ∷ ∙λ ∷ ε ∷ γ ∷ ο ∷ ν ∷ []) "John.7.31"
∷ word (Ὁ ∷ []) "John.7.31"
∷ word (χ ∷ ρ ∷ ι ∷ σ ∷ τ ∷ ὸ ∷ ς ∷ []) "John.7.31"
∷ word (ὅ ∷ τ ∷ α ∷ ν ∷ []) "John.7.31"
∷ word (ἔ ∷ ∙λ ∷ θ ∷ ῃ ∷ []) "John.7.31"
∷ word (μ ∷ ὴ ∷ []) "John.7.31"
∷ word (π ∷ ∙λ ∷ ε ∷ ί ∷ ο ∷ ν ∷ α ∷ []) "John.7.31"
∷ word (σ ∷ η ∷ μ ∷ ε ∷ ῖ ∷ α ∷ []) "John.7.31"
∷ word (π ∷ ο ∷ ι ∷ ή ∷ σ ∷ ε ∷ ι ∷ []) "John.7.31"
∷ word (ὧ ∷ ν ∷ []) "John.7.31"
∷ word (ο ∷ ὗ ∷ τ ∷ ο ∷ ς ∷ []) "John.7.31"
∷ word (ἐ ∷ π ∷ ο ∷ ί ∷ η ∷ σ ∷ ε ∷ ν ∷ []) "John.7.31"
∷ word (Ἤ ∷ κ ∷ ο ∷ υ ∷ σ ∷ α ∷ ν ∷ []) "John.7.32"
∷ word (ο ∷ ἱ ∷ []) "John.7.32"
∷ word (Φ ∷ α ∷ ρ ∷ ι ∷ σ ∷ α ∷ ῖ ∷ ο ∷ ι ∷ []) "John.7.32"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.7.32"
∷ word (ὄ ∷ χ ∷ ∙λ ∷ ο ∷ υ ∷ []) "John.7.32"
∷ word (γ ∷ ο ∷ γ ∷ γ ∷ ύ ∷ ζ ∷ ο ∷ ν ∷ τ ∷ ο ∷ ς ∷ []) "John.7.32"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.7.32"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.7.32"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.7.32"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.7.32"
∷ word (ἀ ∷ π ∷ έ ∷ σ ∷ τ ∷ ε ∷ ι ∷ ∙λ ∷ α ∷ ν ∷ []) "John.7.32"
∷ word (ο ∷ ἱ ∷ []) "John.7.32"
∷ word (ἀ ∷ ρ ∷ χ ∷ ι ∷ ε ∷ ρ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.7.32"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.7.32"
∷ word (ο ∷ ἱ ∷ []) "John.7.32"
∷ word (Φ ∷ α ∷ ρ ∷ ι ∷ σ ∷ α ∷ ῖ ∷ ο ∷ ι ∷ []) "John.7.32"
∷ word (ὑ ∷ π ∷ η ∷ ρ ∷ έ ∷ τ ∷ α ∷ ς ∷ []) "John.7.32"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.7.32"
∷ word (π ∷ ι ∷ ά ∷ σ ∷ ω ∷ σ ∷ ι ∷ ν ∷ []) "John.7.32"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.7.32"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.7.33"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.7.33"
∷ word (ὁ ∷ []) "John.7.33"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.7.33"
∷ word (Ἔ ∷ τ ∷ ι ∷ []) "John.7.33"
∷ word (χ ∷ ρ ∷ ό ∷ ν ∷ ο ∷ ν ∷ []) "John.7.33"
∷ word (μ ∷ ι ∷ κ ∷ ρ ∷ ὸ ∷ ν ∷ []) "John.7.33"
∷ word (μ ∷ ε ∷ θ ∷ []) "John.7.33"
∷ word (ὑ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.7.33"
∷ word (ε ∷ ἰ ∷ μ ∷ ι ∷ []) "John.7.33"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.7.33"
∷ word (ὑ ∷ π ∷ ά ∷ γ ∷ ω ∷ []) "John.7.33"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.7.33"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.7.33"
∷ word (π ∷ έ ∷ μ ∷ ψ ∷ α ∷ ν ∷ τ ∷ ά ∷ []) "John.7.33"
∷ word (μ ∷ ε ∷ []) "John.7.33"
∷ word (ζ ∷ η ∷ τ ∷ ή ∷ σ ∷ ε ∷ τ ∷ έ ∷ []) "John.7.34"
∷ word (μ ∷ ε ∷ []) "John.7.34"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.7.34"
∷ word (ο ∷ ὐ ∷ χ ∷ []) "John.7.34"
∷ word (ε ∷ ὑ ∷ ρ ∷ ή ∷ σ ∷ ε ∷ τ ∷ έ ∷ []) "John.7.34"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.7.34"
∷ word (ὅ ∷ π ∷ ο ∷ υ ∷ []) "John.7.34"
∷ word (ε ∷ ἰ ∷ μ ∷ ὶ ∷ []) "John.7.34"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.7.34"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.7.34"
∷ word (ο ∷ ὐ ∷ []) "John.7.34"
∷ word (δ ∷ ύ ∷ ν ∷ α ∷ σ ∷ θ ∷ ε ∷ []) "John.7.34"
∷ word (ἐ ∷ ∙λ ∷ θ ∷ ε ∷ ῖ ∷ ν ∷ []) "John.7.34"
∷ word (ε ∷ ἶ ∷ π ∷ ο ∷ ν ∷ []) "John.7.35"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.7.35"
∷ word (ο ∷ ἱ ∷ []) "John.7.35"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ῖ ∷ ο ∷ ι ∷ []) "John.7.35"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.7.35"
∷ word (ἑ ∷ α ∷ υ ∷ τ ∷ ο ∷ ύ ∷ ς ∷ []) "John.7.35"
∷ word (Π ∷ ο ∷ ῦ ∷ []) "John.7.35"
∷ word (ο ∷ ὗ ∷ τ ∷ ο ∷ ς ∷ []) "John.7.35"
∷ word (μ ∷ έ ∷ ∙λ ∷ ∙λ ∷ ε ∷ ι ∷ []) "John.7.35"
∷ word (π ∷ ο ∷ ρ ∷ ε ∷ ύ ∷ ε ∷ σ ∷ θ ∷ α ∷ ι ∷ []) "John.7.35"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.7.35"
∷ word (ἡ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.7.35"
∷ word (ο ∷ ὐ ∷ χ ∷ []) "John.7.35"
∷ word (ε ∷ ὑ ∷ ρ ∷ ή ∷ σ ∷ ο ∷ μ ∷ ε ∷ ν ∷ []) "John.7.35"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.7.35"
∷ word (μ ∷ ὴ ∷ []) "John.7.35"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.7.35"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.7.35"
∷ word (δ ∷ ι ∷ α ∷ σ ∷ π ∷ ο ∷ ρ ∷ ὰ ∷ ν ∷ []) "John.7.35"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.7.35"
∷ word (Ἑ ∷ ∙λ ∷ ∙λ ∷ ή ∷ ν ∷ ω ∷ ν ∷ []) "John.7.35"
∷ word (μ ∷ έ ∷ ∙λ ∷ ∙λ ∷ ε ∷ ι ∷ []) "John.7.35"
∷ word (π ∷ ο ∷ ρ ∷ ε ∷ ύ ∷ ε ∷ σ ∷ θ ∷ α ∷ ι ∷ []) "John.7.35"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.7.35"
∷ word (δ ∷ ι ∷ δ ∷ ά ∷ σ ∷ κ ∷ ε ∷ ι ∷ ν ∷ []) "John.7.35"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.7.35"
∷ word (Ἕ ∷ ∙λ ∷ ∙λ ∷ η ∷ ν ∷ α ∷ ς ∷ []) "John.7.35"
∷ word (τ ∷ ί ∷ ς ∷ []) "John.7.36"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.7.36"
∷ word (ὁ ∷ []) "John.7.36"
∷ word (∙λ ∷ ό ∷ γ ∷ ο ∷ ς ∷ []) "John.7.36"
∷ word (ο ∷ ὗ ∷ τ ∷ ο ∷ ς ∷ []) "John.7.36"
∷ word (ὃ ∷ ν ∷ []) "John.7.36"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ []) "John.7.36"
∷ word (Ζ ∷ η ∷ τ ∷ ή ∷ σ ∷ ε ∷ τ ∷ έ ∷ []) "John.7.36"
∷ word (μ ∷ ε ∷ []) "John.7.36"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.7.36"
∷ word (ο ∷ ὐ ∷ χ ∷ []) "John.7.36"
∷ word (ε ∷ ὑ ∷ ρ ∷ ή ∷ σ ∷ ε ∷ τ ∷ έ ∷ []) "John.7.36"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.7.36"
∷ word (ὅ ∷ π ∷ ο ∷ υ ∷ []) "John.7.36"
∷ word (ε ∷ ἰ ∷ μ ∷ ὶ ∷ []) "John.7.36"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.7.36"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.7.36"
∷ word (ο ∷ ὐ ∷ []) "John.7.36"
∷ word (δ ∷ ύ ∷ ν ∷ α ∷ σ ∷ θ ∷ ε ∷ []) "John.7.36"
∷ word (ἐ ∷ ∙λ ∷ θ ∷ ε ∷ ῖ ∷ ν ∷ []) "John.7.36"
∷ word (Ἐ ∷ ν ∷ []) "John.7.37"
∷ word (δ ∷ ὲ ∷ []) "John.7.37"
∷ word (τ ∷ ῇ ∷ []) "John.7.37"
∷ word (ἐ ∷ σ ∷ χ ∷ ά ∷ τ ∷ ῃ ∷ []) "John.7.37"
∷ word (ἡ ∷ μ ∷ έ ∷ ρ ∷ ᾳ ∷ []) "John.7.37"
∷ word (τ ∷ ῇ ∷ []) "John.7.37"
∷ word (μ ∷ ε ∷ γ ∷ ά ∷ ∙λ ∷ ῃ ∷ []) "John.7.37"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.7.37"
∷ word (ἑ ∷ ο ∷ ρ ∷ τ ∷ ῆ ∷ ς ∷ []) "John.7.37"
∷ word (ε ∷ ἱ ∷ σ ∷ τ ∷ ή ∷ κ ∷ ε ∷ ι ∷ []) "John.7.37"
∷ word (ὁ ∷ []) "John.7.37"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.7.37"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.7.37"
∷ word (ἔ ∷ κ ∷ ρ ∷ α ∷ ξ ∷ ε ∷ ν ∷ []) "John.7.37"
∷ word (∙λ ∷ έ ∷ γ ∷ ω ∷ ν ∷ []) "John.7.37"
∷ word (Ἐ ∷ ά ∷ ν ∷ []) "John.7.37"
∷ word (τ ∷ ι ∷ ς ∷ []) "John.7.37"
∷ word (δ ∷ ι ∷ ψ ∷ ᾷ ∷ []) "John.7.37"
∷ word (ἐ ∷ ρ ∷ χ ∷ έ ∷ σ ∷ θ ∷ ω ∷ []) "John.7.37"
∷ word (π ∷ ρ ∷ ό ∷ ς ∷ []) "John.7.37"
∷ word (μ ∷ ε ∷ []) "John.7.37"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.7.37"
∷ word (π ∷ ι ∷ ν ∷ έ ∷ τ ∷ ω ∷ []) "John.7.37"
∷ word (ὁ ∷ []) "John.7.38"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ ω ∷ ν ∷ []) "John.7.38"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.7.38"
∷ word (ἐ ∷ μ ∷ έ ∷ []) "John.7.38"
∷ word (κ ∷ α ∷ θ ∷ ὼ ∷ ς ∷ []) "John.7.38"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.7.38"
∷ word (ἡ ∷ []) "John.7.38"
∷ word (γ ∷ ρ ∷ α ∷ φ ∷ ή ∷ []) "John.7.38"
∷ word (π ∷ ο ∷ τ ∷ α ∷ μ ∷ ο ∷ ὶ ∷ []) "John.7.38"
∷ word (ἐ ∷ κ ∷ []) "John.7.38"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.7.38"
∷ word (κ ∷ ο ∷ ι ∷ ∙λ ∷ ί ∷ α ∷ ς ∷ []) "John.7.38"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.7.38"
∷ word (ῥ ∷ ε ∷ ύ ∷ σ ∷ ο ∷ υ ∷ σ ∷ ι ∷ ν ∷ []) "John.7.38"
∷ word (ὕ ∷ δ ∷ α ∷ τ ∷ ο ∷ ς ∷ []) "John.7.38"
∷ word (ζ ∷ ῶ ∷ ν ∷ τ ∷ ο ∷ ς ∷ []) "John.7.38"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.7.39"
∷ word (δ ∷ ὲ ∷ []) "John.7.39"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.7.39"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.7.39"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.7.39"
∷ word (π ∷ ν ∷ ε ∷ ύ ∷ μ ∷ α ∷ τ ∷ ο ∷ ς ∷ []) "John.7.39"
∷ word (ο ∷ ὗ ∷ []) "John.7.39"
∷ word (ἔ ∷ μ ∷ ε ∷ ∙λ ∷ ∙λ ∷ ο ∷ ν ∷ []) "John.7.39"
∷ word (∙λ ∷ α ∷ μ ∷ β ∷ ά ∷ ν ∷ ε ∷ ι ∷ ν ∷ []) "John.7.39"
∷ word (ο ∷ ἱ ∷ []) "John.7.39"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ σ ∷ α ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.7.39"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.7.39"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.7.39"
∷ word (ο ∷ ὔ ∷ π ∷ ω ∷ []) "John.7.39"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.7.39"
∷ word (ἦ ∷ ν ∷ []) "John.7.39"
∷ word (π ∷ ν ∷ ε ∷ ῦ ∷ μ ∷ α ∷ []) "John.7.39"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.7.39"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.7.39"
∷ word (ο ∷ ὐ ∷ δ ∷ έ ∷ π ∷ ω ∷ []) "John.7.39"
∷ word (ἐ ∷ δ ∷ ο ∷ ξ ∷ ά ∷ σ ∷ θ ∷ η ∷ []) "John.7.39"
∷ word (Ἐ ∷ κ ∷ []) "John.7.40"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.7.40"
∷ word (ὄ ∷ χ ∷ ∙λ ∷ ο ∷ υ ∷ []) "John.7.40"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.7.40"
∷ word (ἀ ∷ κ ∷ ο ∷ ύ ∷ σ ∷ α ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.7.40"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.7.40"
∷ word (∙λ ∷ ό ∷ γ ∷ ω ∷ ν ∷ []) "John.7.40"
∷ word (τ ∷ ο ∷ ύ ∷ τ ∷ ω ∷ ν ∷ []) "John.7.40"
∷ word (ἔ ∷ ∙λ ∷ ε ∷ γ ∷ ο ∷ ν ∷ []) "John.7.40"
∷ word (Ο ∷ ὗ ∷ τ ∷ ό ∷ ς ∷ []) "John.7.40"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.7.40"
∷ word (ἀ ∷ ∙λ ∷ η ∷ θ ∷ ῶ ∷ ς ∷ []) "John.7.40"
∷ word (ὁ ∷ []) "John.7.40"
∷ word (π ∷ ρ ∷ ο ∷ φ ∷ ή ∷ τ ∷ η ∷ ς ∷ []) "John.7.40"
∷ word (ἄ ∷ ∙λ ∷ ∙λ ∷ ο ∷ ι ∷ []) "John.7.41"
∷ word (ἔ ∷ ∙λ ∷ ε ∷ γ ∷ ο ∷ ν ∷ []) "John.7.41"
∷ word (Ο ∷ ὗ ∷ τ ∷ ό ∷ ς ∷ []) "John.7.41"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.7.41"
∷ word (ὁ ∷ []) "John.7.41"
∷ word (χ ∷ ρ ∷ ι ∷ σ ∷ τ ∷ ό ∷ ς ∷ []) "John.7.41"
∷ word (ο ∷ ἱ ∷ []) "John.7.41"
∷ word (δ ∷ ὲ ∷ []) "John.7.41"
∷ word (ἔ ∷ ∙λ ∷ ε ∷ γ ∷ ο ∷ ν ∷ []) "John.7.41"
∷ word (Μ ∷ ὴ ∷ []) "John.7.41"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.7.41"
∷ word (ἐ ∷ κ ∷ []) "John.7.41"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.7.41"
∷ word (Γ ∷ α ∷ ∙λ ∷ ι ∷ ∙λ ∷ α ∷ ί ∷ α ∷ ς ∷ []) "John.7.41"
∷ word (ὁ ∷ []) "John.7.41"
∷ word (χ ∷ ρ ∷ ι ∷ σ ∷ τ ∷ ὸ ∷ ς ∷ []) "John.7.41"
∷ word (ἔ ∷ ρ ∷ χ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.7.41"
∷ word (ο ∷ ὐ ∷ χ ∷ []) "John.7.42"
∷ word (ἡ ∷ []) "John.7.42"
∷ word (γ ∷ ρ ∷ α ∷ φ ∷ ὴ ∷ []) "John.7.42"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.7.42"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.7.42"
∷ word (ἐ ∷ κ ∷ []) "John.7.42"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.7.42"
∷ word (σ ∷ π ∷ έ ∷ ρ ∷ μ ∷ α ∷ τ ∷ ο ∷ ς ∷ []) "John.7.42"
∷ word (Δ ∷ α ∷ υ ∷ ὶ ∷ δ ∷ []) "John.7.42"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.7.42"
∷ word (ἀ ∷ π ∷ ὸ ∷ []) "John.7.42"
∷ word (Β ∷ η ∷ θ ∷ ∙λ ∷ έ ∷ ε ∷ μ ∷ []) "John.7.42"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.7.42"
∷ word (κ ∷ ώ ∷ μ ∷ η ∷ ς ∷ []) "John.7.42"
∷ word (ὅ ∷ π ∷ ο ∷ υ ∷ []) "John.7.42"
∷ word (ἦ ∷ ν ∷ []) "John.7.42"
∷ word (Δ ∷ α ∷ υ ∷ ὶ ∷ δ ∷ []) "John.7.42"
∷ word (ἔ ∷ ρ ∷ χ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.7.42"
∷ word (ὁ ∷ []) "John.7.42"
∷ word (χ ∷ ρ ∷ ι ∷ σ ∷ τ ∷ ό ∷ ς ∷ []) "John.7.42"
∷ word (σ ∷ χ ∷ ί ∷ σ ∷ μ ∷ α ∷ []) "John.7.43"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.7.43"
∷ word (ἐ ∷ γ ∷ έ ∷ ν ∷ ε ∷ τ ∷ ο ∷ []) "John.7.43"
∷ word (ἐ ∷ ν ∷ []) "John.7.43"
∷ word (τ ∷ ῷ ∷ []) "John.7.43"
∷ word (ὄ ∷ χ ∷ ∙λ ∷ ῳ ∷ []) "John.7.43"
∷ word (δ ∷ ι ∷ []) "John.7.43"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.7.43"
∷ word (τ ∷ ι ∷ ν ∷ ὲ ∷ ς ∷ []) "John.7.44"
∷ word (δ ∷ ὲ ∷ []) "John.7.44"
∷ word (ἤ ∷ θ ∷ ε ∷ ∙λ ∷ ο ∷ ν ∷ []) "John.7.44"
∷ word (ἐ ∷ ξ ∷ []) "John.7.44"
∷ word (α ∷ ὐ ∷ τ ∷ ῶ ∷ ν ∷ []) "John.7.44"
∷ word (π ∷ ι ∷ ά ∷ σ ∷ α ∷ ι ∷ []) "John.7.44"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.7.44"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ []) "John.7.44"
∷ word (ο ∷ ὐ ∷ δ ∷ ε ∷ ὶ ∷ ς ∷ []) "John.7.44"
∷ word (ἐ ∷ π ∷ έ ∷ β ∷ α ∷ ∙λ ∷ ε ∷ ν ∷ []) "John.7.44"
∷ word (ἐ ∷ π ∷ []) "John.7.44"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.7.44"
∷ word (τ ∷ ὰ ∷ ς ∷ []) "John.7.44"
∷ word (χ ∷ ε ∷ ῖ ∷ ρ ∷ α ∷ ς ∷ []) "John.7.44"
∷ word (Ἦ ∷ ∙λ ∷ θ ∷ ο ∷ ν ∷ []) "John.7.45"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.7.45"
∷ word (ο ∷ ἱ ∷ []) "John.7.45"
∷ word (ὑ ∷ π ∷ η ∷ ρ ∷ έ ∷ τ ∷ α ∷ ι ∷ []) "John.7.45"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.7.45"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.7.45"
∷ word (ἀ ∷ ρ ∷ χ ∷ ι ∷ ε ∷ ρ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.7.45"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.7.45"
∷ word (Φ ∷ α ∷ ρ ∷ ι ∷ σ ∷ α ∷ ί ∷ ο ∷ υ ∷ ς ∷ []) "John.7.45"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.7.45"
∷ word (ε ∷ ἶ ∷ π ∷ ο ∷ ν ∷ []) "John.7.45"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.7.45"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ο ∷ ι ∷ []) "John.7.45"
∷ word (Δ ∷ ι ∷ ὰ ∷ []) "John.7.45"
∷ word (τ ∷ ί ∷ []) "John.7.45"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.7.45"
∷ word (ἠ ∷ γ ∷ ά ∷ γ ∷ ε ∷ τ ∷ ε ∷ []) "John.7.45"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.7.45"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.7.46"
∷ word (ο ∷ ἱ ∷ []) "John.7.46"
∷ word (ὑ ∷ π ∷ η ∷ ρ ∷ έ ∷ τ ∷ α ∷ ι ∷ []) "John.7.46"
∷ word (Ο ∷ ὐ ∷ δ ∷ έ ∷ π ∷ ο ∷ τ ∷ ε ∷ []) "John.7.46"
∷ word (ἐ ∷ ∙λ ∷ ά ∷ ∙λ ∷ η ∷ σ ∷ ε ∷ ν ∷ []) "John.7.46"
∷ word (ο ∷ ὕ ∷ τ ∷ ω ∷ ς ∷ []) "John.7.46"
∷ word (ἄ ∷ ν ∷ θ ∷ ρ ∷ ω ∷ π ∷ ο ∷ ς ∷ []) "John.7.46"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.7.47"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.7.47"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.7.47"
∷ word (ο ∷ ἱ ∷ []) "John.7.47"
∷ word (Φ ∷ α ∷ ρ ∷ ι ∷ σ ∷ α ∷ ῖ ∷ ο ∷ ι ∷ []) "John.7.47"
∷ word (Μ ∷ ὴ ∷ []) "John.7.47"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.7.47"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.7.47"
∷ word (π ∷ ε ∷ π ∷ ∙λ ∷ ά ∷ ν ∷ η ∷ σ ∷ θ ∷ ε ∷ []) "John.7.47"
∷ word (μ ∷ ή ∷ []) "John.7.48"
∷ word (τ ∷ ι ∷ ς ∷ []) "John.7.48"
∷ word (ἐ ∷ κ ∷ []) "John.7.48"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.7.48"
∷ word (ἀ ∷ ρ ∷ χ ∷ ό ∷ ν ∷ τ ∷ ω ∷ ν ∷ []) "John.7.48"
∷ word (ἐ ∷ π ∷ ί ∷ σ ∷ τ ∷ ε ∷ υ ∷ σ ∷ ε ∷ ν ∷ []) "John.7.48"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.7.48"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.7.48"
∷ word (ἢ ∷ []) "John.7.48"
∷ word (ἐ ∷ κ ∷ []) "John.7.48"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.7.48"
∷ word (Φ ∷ α ∷ ρ ∷ ι ∷ σ ∷ α ∷ ί ∷ ω ∷ ν ∷ []) "John.7.48"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.7.49"
∷ word (ὁ ∷ []) "John.7.49"
∷ word (ὄ ∷ χ ∷ ∙λ ∷ ο ∷ ς ∷ []) "John.7.49"
∷ word (ο ∷ ὗ ∷ τ ∷ ο ∷ ς ∷ []) "John.7.49"
∷ word (ὁ ∷ []) "John.7.49"
∷ word (μ ∷ ὴ ∷ []) "John.7.49"
∷ word (γ ∷ ι ∷ ν ∷ ώ ∷ σ ∷ κ ∷ ω ∷ ν ∷ []) "John.7.49"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.7.49"
∷ word (ν ∷ ό ∷ μ ∷ ο ∷ ν ∷ []) "John.7.49"
∷ word (ἐ ∷ π ∷ ά ∷ ρ ∷ α ∷ τ ∷ ο ∷ ί ∷ []) "John.7.49"
∷ word (ε ∷ ἰ ∷ σ ∷ ι ∷ ν ∷ []) "John.7.49"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.7.50"
∷ word (Ν ∷ ι ∷ κ ∷ ό ∷ δ ∷ η ∷ μ ∷ ο ∷ ς ∷ []) "John.7.50"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.7.50"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ύ ∷ ς ∷ []) "John.7.50"
∷ word (ὁ ∷ []) "John.7.50"
∷ word (ἐ ∷ ∙λ ∷ θ ∷ ὼ ∷ ν ∷ []) "John.7.50"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.7.50"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.7.50"
∷ word (π ∷ ρ ∷ ό ∷ τ ∷ ε ∷ ρ ∷ ο ∷ ν ∷ []) "John.7.50"
∷ word (ε ∷ ἷ ∷ ς ∷ []) "John.7.50"
∷ word (ὢ ∷ ν ∷ []) "John.7.50"
∷ word (ἐ ∷ ξ ∷ []) "John.7.50"
∷ word (α ∷ ὐ ∷ τ ∷ ῶ ∷ ν ∷ []) "John.7.50"
∷ word (Μ ∷ ὴ ∷ []) "John.7.51"
∷ word (ὁ ∷ []) "John.7.51"
∷ word (ν ∷ ό ∷ μ ∷ ο ∷ ς ∷ []) "John.7.51"
∷ word (ἡ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.7.51"
∷ word (κ ∷ ρ ∷ ί ∷ ν ∷ ε ∷ ι ∷ []) "John.7.51"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.7.51"
∷ word (ἄ ∷ ν ∷ θ ∷ ρ ∷ ω ∷ π ∷ ο ∷ ν ∷ []) "John.7.51"
∷ word (ἐ ∷ ὰ ∷ ν ∷ []) "John.7.51"
∷ word (μ ∷ ὴ ∷ []) "John.7.51"
∷ word (ἀ ∷ κ ∷ ο ∷ ύ ∷ σ ∷ ῃ ∷ []) "John.7.51"
∷ word (π ∷ ρ ∷ ῶ ∷ τ ∷ ο ∷ ν ∷ []) "John.7.51"
∷ word (π ∷ α ∷ ρ ∷ []) "John.7.51"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.7.51"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.7.51"
∷ word (γ ∷ ν ∷ ῷ ∷ []) "John.7.51"
∷ word (τ ∷ ί ∷ []) "John.7.51"
∷ word (π ∷ ο ∷ ι ∷ ε ∷ ῖ ∷ []) "John.7.51"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.7.52"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.7.52"
∷ word (ε ∷ ἶ ∷ π ∷ α ∷ ν ∷ []) "John.7.52"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.7.52"
∷ word (Μ ∷ ὴ ∷ []) "John.7.52"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.7.52"
∷ word (σ ∷ ὺ ∷ []) "John.7.52"
∷ word (ἐ ∷ κ ∷ []) "John.7.52"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.7.52"
∷ word (Γ ∷ α ∷ ∙λ ∷ ι ∷ ∙λ ∷ α ∷ ί ∷ α ∷ ς ∷ []) "John.7.52"
∷ word (ε ∷ ἶ ∷ []) "John.7.52"
∷ word (ἐ ∷ ρ ∷ α ∷ ύ ∷ ν ∷ η ∷ σ ∷ ο ∷ ν ∷ []) "John.7.52"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.7.52"
∷ word (ἴ ∷ δ ∷ ε ∷ []) "John.7.52"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.7.52"
∷ word (ἐ ∷ κ ∷ []) "John.7.52"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.7.52"
∷ word (Γ ∷ α ∷ ∙λ ∷ ι ∷ ∙λ ∷ α ∷ ί ∷ α ∷ ς ∷ []) "John.7.52"
∷ word (π ∷ ρ ∷ ο ∷ φ ∷ ή ∷ τ ∷ η ∷ ς ∷ []) "John.7.52"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.7.52"
∷ word (ἐ ∷ γ ∷ ε ∷ ί ∷ ρ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.7.52"
∷ word (Π ∷ ά ∷ ∙λ ∷ ι ∷ ν ∷ []) "John.8.12"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.8.12"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.8.12"
∷ word (ἐ ∷ ∙λ ∷ ά ∷ ∙λ ∷ η ∷ σ ∷ ε ∷ ν ∷ []) "John.8.12"
∷ word (ὁ ∷ []) "John.8.12"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.8.12"
∷ word (∙λ ∷ έ ∷ γ ∷ ω ∷ ν ∷ []) "John.8.12"
∷ word (Ἐ ∷ γ ∷ ώ ∷ []) "John.8.12"
∷ word (ε ∷ ἰ ∷ μ ∷ ι ∷ []) "John.8.12"
∷ word (τ ∷ ὸ ∷ []) "John.8.12"
∷ word (φ ∷ ῶ ∷ ς ∷ []) "John.8.12"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.8.12"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ υ ∷ []) "John.8.12"
∷ word (ὁ ∷ []) "John.8.12"
∷ word (ἀ ∷ κ ∷ ο ∷ ∙λ ∷ ο ∷ υ ∷ θ ∷ ῶ ∷ ν ∷ []) "John.8.12"
∷ word (ἐ ∷ μ ∷ ο ∷ ὶ ∷ []) "John.8.12"
∷ word (ο ∷ ὐ ∷ []) "John.8.12"
∷ word (μ ∷ ὴ ∷ []) "John.8.12"
∷ word (π ∷ ε ∷ ρ ∷ ι ∷ π ∷ α ∷ τ ∷ ή ∷ σ ∷ ῃ ∷ []) "John.8.12"
∷ word (ἐ ∷ ν ∷ []) "John.8.12"
∷ word (τ ∷ ῇ ∷ []) "John.8.12"
∷ word (σ ∷ κ ∷ ο ∷ τ ∷ ί ∷ ᾳ ∷ []) "John.8.12"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ []) "John.8.12"
∷ word (ἕ ∷ ξ ∷ ε ∷ ι ∷ []) "John.8.12"
∷ word (τ ∷ ὸ ∷ []) "John.8.12"
∷ word (φ ∷ ῶ ∷ ς ∷ []) "John.8.12"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.8.12"
∷ word (ζ ∷ ω ∷ ῆ ∷ ς ∷ []) "John.8.12"
∷ word (ε ∷ ἶ ∷ π ∷ ο ∷ ν ∷ []) "John.8.13"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.8.13"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.8.13"
∷ word (ο ∷ ἱ ∷ []) "John.8.13"
∷ word (Φ ∷ α ∷ ρ ∷ ι ∷ σ ∷ α ∷ ῖ ∷ ο ∷ ι ∷ []) "John.8.13"
∷ word (Σ ∷ ὺ ∷ []) "John.8.13"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.8.13"
∷ word (σ ∷ ε ∷ α ∷ υ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.8.13"
∷ word (μ ∷ α ∷ ρ ∷ τ ∷ υ ∷ ρ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.8.13"
∷ word (ἡ ∷ []) "John.8.13"
∷ word (μ ∷ α ∷ ρ ∷ τ ∷ υ ∷ ρ ∷ ί ∷ α ∷ []) "John.8.13"
∷ word (σ ∷ ο ∷ υ ∷ []) "John.8.13"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.8.13"
∷ word (ἔ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.8.13"
∷ word (ἀ ∷ ∙λ ∷ η ∷ θ ∷ ή ∷ ς ∷ []) "John.8.13"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.8.14"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.8.14"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.8.14"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.8.14"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.8.14"
∷ word (Κ ∷ ἂ ∷ ν ∷ []) "John.8.14"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.8.14"
∷ word (μ ∷ α ∷ ρ ∷ τ ∷ υ ∷ ρ ∷ ῶ ∷ []) "John.8.14"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.8.14"
∷ word (ἐ ∷ μ ∷ α ∷ υ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.8.14"
∷ word (ἀ ∷ ∙λ ∷ η ∷ θ ∷ ή ∷ ς ∷ []) "John.8.14"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.8.14"
∷ word (ἡ ∷ []) "John.8.14"
∷ word (μ ∷ α ∷ ρ ∷ τ ∷ υ ∷ ρ ∷ ί ∷ α ∷ []) "John.8.14"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.8.14"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.8.14"
∷ word (ο ∷ ἶ ∷ δ ∷ α ∷ []) "John.8.14"
∷ word (π ∷ ό ∷ θ ∷ ε ∷ ν ∷ []) "John.8.14"
∷ word (ἦ ∷ ∙λ ∷ θ ∷ ο ∷ ν ∷ []) "John.8.14"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.8.14"
∷ word (π ∷ ο ∷ ῦ ∷ []) "John.8.14"
∷ word (ὑ ∷ π ∷ ά ∷ γ ∷ ω ∷ []) "John.8.14"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.8.14"
∷ word (δ ∷ ὲ ∷ []) "John.8.14"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.8.14"
∷ word (ο ∷ ἴ ∷ δ ∷ α ∷ τ ∷ ε ∷ []) "John.8.14"
∷ word (π ∷ ό ∷ θ ∷ ε ∷ ν ∷ []) "John.8.14"
∷ word (ἔ ∷ ρ ∷ χ ∷ ο ∷ μ ∷ α ∷ ι ∷ []) "John.8.14"
∷ word (ἢ ∷ []) "John.8.14"
∷ word (π ∷ ο ∷ ῦ ∷ []) "John.8.14"
∷ word (ὑ ∷ π ∷ ά ∷ γ ∷ ω ∷ []) "John.8.14"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.8.15"
∷ word (κ ∷ α ∷ τ ∷ ὰ ∷ []) "John.8.15"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.8.15"
∷ word (σ ∷ ά ∷ ρ ∷ κ ∷ α ∷ []) "John.8.15"
∷ word (κ ∷ ρ ∷ ί ∷ ν ∷ ε ∷ τ ∷ ε ∷ []) "John.8.15"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.8.15"
∷ word (ο ∷ ὐ ∷ []) "John.8.15"
∷ word (κ ∷ ρ ∷ ί ∷ ν ∷ ω ∷ []) "John.8.15"
∷ word (ο ∷ ὐ ∷ δ ∷ έ ∷ ν ∷ α ∷ []) "John.8.15"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.8.16"
∷ word (ἐ ∷ ὰ ∷ ν ∷ []) "John.8.16"
∷ word (κ ∷ ρ ∷ ί ∷ ν ∷ ω ∷ []) "John.8.16"
∷ word (δ ∷ ὲ ∷ []) "John.8.16"
∷ word (ἐ ∷ γ ∷ ώ ∷ []) "John.8.16"
∷ word (ἡ ∷ []) "John.8.16"
∷ word (κ ∷ ρ ∷ ί ∷ σ ∷ ι ∷ ς ∷ []) "John.8.16"
∷ word (ἡ ∷ []) "John.8.16"
∷ word (ἐ ∷ μ ∷ ὴ ∷ []) "John.8.16"
∷ word (ἀ ∷ ∙λ ∷ η ∷ θ ∷ ι ∷ ν ∷ ή ∷ []) "John.8.16"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.8.16"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.8.16"
∷ word (μ ∷ ό ∷ ν ∷ ο ∷ ς ∷ []) "John.8.16"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.8.16"
∷ word (ε ∷ ἰ ∷ μ ∷ ί ∷ []) "John.8.16"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ []) "John.8.16"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.8.16"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.8.16"
∷ word (ὁ ∷ []) "John.8.16"
∷ word (π ∷ έ ∷ μ ∷ ψ ∷ α ∷ ς ∷ []) "John.8.16"
∷ word (μ ∷ ε ∷ []) "John.8.16"
∷ word (π ∷ α ∷ τ ∷ ή ∷ ρ ∷ []) "John.8.16"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.8.17"
∷ word (ἐ ∷ ν ∷ []) "John.8.17"
∷ word (τ ∷ ῷ ∷ []) "John.8.17"
∷ word (ν ∷ ό ∷ μ ∷ ῳ ∷ []) "John.8.17"
∷ word (δ ∷ ὲ ∷ []) "John.8.17"
∷ word (τ ∷ ῷ ∷ []) "John.8.17"
∷ word (ὑ ∷ μ ∷ ε ∷ τ ∷ έ ∷ ρ ∷ ῳ ∷ []) "John.8.17"
∷ word (γ ∷ έ ∷ γ ∷ ρ ∷ α ∷ π ∷ τ ∷ α ∷ ι ∷ []) "John.8.17"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.8.17"
∷ word (δ ∷ ύ ∷ ο ∷ []) "John.8.17"
∷ word (ἀ ∷ ν ∷ θ ∷ ρ ∷ ώ ∷ π ∷ ω ∷ ν ∷ []) "John.8.17"
∷ word (ἡ ∷ []) "John.8.17"
∷ word (μ ∷ α ∷ ρ ∷ τ ∷ υ ∷ ρ ∷ ί ∷ α ∷ []) "John.8.17"
∷ word (ἀ ∷ ∙λ ∷ η ∷ θ ∷ ή ∷ ς ∷ []) "John.8.17"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.8.17"
∷ word (ἐ ∷ γ ∷ ώ ∷ []) "John.8.18"
∷ word (ε ∷ ἰ ∷ μ ∷ ι ∷ []) "John.8.18"
∷ word (ὁ ∷ []) "John.8.18"
∷ word (μ ∷ α ∷ ρ ∷ τ ∷ υ ∷ ρ ∷ ῶ ∷ ν ∷ []) "John.8.18"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.8.18"
∷ word (ἐ ∷ μ ∷ α ∷ υ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.8.18"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.8.18"
∷ word (μ ∷ α ∷ ρ ∷ τ ∷ υ ∷ ρ ∷ ε ∷ ῖ ∷ []) "John.8.18"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.8.18"
∷ word (ἐ ∷ μ ∷ ο ∷ ῦ ∷ []) "John.8.18"
∷ word (ὁ ∷ []) "John.8.18"
∷ word (π ∷ έ ∷ μ ∷ ψ ∷ α ∷ ς ∷ []) "John.8.18"
∷ word (μ ∷ ε ∷ []) "John.8.18"
∷ word (π ∷ α ∷ τ ∷ ή ∷ ρ ∷ []) "John.8.18"
∷ word (ἔ ∷ ∙λ ∷ ε ∷ γ ∷ ο ∷ ν ∷ []) "John.8.19"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.8.19"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.8.19"
∷ word (Π ∷ ο ∷ ῦ ∷ []) "John.8.19"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.8.19"
∷ word (ὁ ∷ []) "John.8.19"
∷ word (π ∷ α ∷ τ ∷ ή ∷ ρ ∷ []) "John.8.19"
∷ word (σ ∷ ο ∷ υ ∷ []) "John.8.19"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.8.19"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.8.19"
∷ word (Ο ∷ ὔ ∷ τ ∷ ε ∷ []) "John.8.19"
∷ word (ἐ ∷ μ ∷ ὲ ∷ []) "John.8.19"
∷ word (ο ∷ ἴ ∷ δ ∷ α ∷ τ ∷ ε ∷ []) "John.8.19"
∷ word (ο ∷ ὔ ∷ τ ∷ ε ∷ []) "John.8.19"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.8.19"
∷ word (π ∷ α ∷ τ ∷ έ ∷ ρ ∷ α ∷ []) "John.8.19"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.8.19"
∷ word (ε ∷ ἰ ∷ []) "John.8.19"
∷ word (ἐ ∷ μ ∷ ὲ ∷ []) "John.8.19"
∷ word (ᾔ ∷ δ ∷ ε ∷ ι ∷ τ ∷ ε ∷ []) "John.8.19"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.8.19"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.8.19"
∷ word (π ∷ α ∷ τ ∷ έ ∷ ρ ∷ α ∷ []) "John.8.19"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.8.19"
∷ word (ἂ ∷ ν ∷ []) "John.8.19"
∷ word (ᾔ ∷ δ ∷ ε ∷ ι ∷ τ ∷ ε ∷ []) "John.8.19"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.8.20"
∷ word (τ ∷ ὰ ∷ []) "John.8.20"
∷ word (ῥ ∷ ή ∷ μ ∷ α ∷ τ ∷ α ∷ []) "John.8.20"
∷ word (ἐ ∷ ∙λ ∷ ά ∷ ∙λ ∷ η ∷ σ ∷ ε ∷ ν ∷ []) "John.8.20"
∷ word (ἐ ∷ ν ∷ []) "John.8.20"
∷ word (τ ∷ ῷ ∷ []) "John.8.20"
∷ word (γ ∷ α ∷ ζ ∷ ο ∷ φ ∷ υ ∷ ∙λ ∷ α ∷ κ ∷ ί ∷ ῳ ∷ []) "John.8.20"
∷ word (δ ∷ ι ∷ δ ∷ ά ∷ σ ∷ κ ∷ ω ∷ ν ∷ []) "John.8.20"
∷ word (ἐ ∷ ν ∷ []) "John.8.20"
∷ word (τ ∷ ῷ ∷ []) "John.8.20"
∷ word (ἱ ∷ ε ∷ ρ ∷ ῷ ∷ []) "John.8.20"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.8.20"
∷ word (ο ∷ ὐ ∷ δ ∷ ε ∷ ὶ ∷ ς ∷ []) "John.8.20"
∷ word (ἐ ∷ π ∷ ί ∷ α ∷ σ ∷ ε ∷ ν ∷ []) "John.8.20"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.8.20"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.8.20"
∷ word (ο ∷ ὔ ∷ π ∷ ω ∷ []) "John.8.20"
∷ word (ἐ ∷ ∙λ ∷ η ∷ ∙λ ∷ ύ ∷ θ ∷ ε ∷ ι ∷ []) "John.8.20"
∷ word (ἡ ∷ []) "John.8.20"
∷ word (ὥ ∷ ρ ∷ α ∷ []) "John.8.20"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.8.20"
∷ word (Ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.8.21"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.8.21"
∷ word (π ∷ ά ∷ ∙λ ∷ ι ∷ ν ∷ []) "John.8.21"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.8.21"
∷ word (Ἐ ∷ γ ∷ ὼ ∷ []) "John.8.21"
∷ word (ὑ ∷ π ∷ ά ∷ γ ∷ ω ∷ []) "John.8.21"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.8.21"
∷ word (ζ ∷ η ∷ τ ∷ ή ∷ σ ∷ ε ∷ τ ∷ έ ∷ []) "John.8.21"
∷ word (μ ∷ ε ∷ []) "John.8.21"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.8.21"
∷ word (ἐ ∷ ν ∷ []) "John.8.21"
∷ word (τ ∷ ῇ ∷ []) "John.8.21"
∷ word (ἁ ∷ μ ∷ α ∷ ρ ∷ τ ∷ ί ∷ ᾳ ∷ []) "John.8.21"
∷ word (ὑ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.8.21"
∷ word (ἀ ∷ π ∷ ο ∷ θ ∷ α ∷ ν ∷ ε ∷ ῖ ∷ σ ∷ θ ∷ ε ∷ []) "John.8.21"
∷ word (ὅ ∷ π ∷ ο ∷ υ ∷ []) "John.8.21"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.8.21"
∷ word (ὑ ∷ π ∷ ά ∷ γ ∷ ω ∷ []) "John.8.21"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.8.21"
∷ word (ο ∷ ὐ ∷ []) "John.8.21"
∷ word (δ ∷ ύ ∷ ν ∷ α ∷ σ ∷ θ ∷ ε ∷ []) "John.8.21"
∷ word (ἐ ∷ ∙λ ∷ θ ∷ ε ∷ ῖ ∷ ν ∷ []) "John.8.21"
∷ word (ἔ ∷ ∙λ ∷ ε ∷ γ ∷ ο ∷ ν ∷ []) "John.8.22"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.8.22"
∷ word (ο ∷ ἱ ∷ []) "John.8.22"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ῖ ∷ ο ∷ ι ∷ []) "John.8.22"
∷ word (Μ ∷ ή ∷ τ ∷ ι ∷ []) "John.8.22"
∷ word (ἀ ∷ π ∷ ο ∷ κ ∷ τ ∷ ε ∷ ν ∷ ε ∷ ῖ ∷ []) "John.8.22"
∷ word (ἑ ∷ α ∷ υ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.8.22"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.8.22"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.8.22"
∷ word (Ὅ ∷ π ∷ ο ∷ υ ∷ []) "John.8.22"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.8.22"
∷ word (ὑ ∷ π ∷ ά ∷ γ ∷ ω ∷ []) "John.8.22"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.8.22"
∷ word (ο ∷ ὐ ∷ []) "John.8.22"
∷ word (δ ∷ ύ ∷ ν ∷ α ∷ σ ∷ θ ∷ ε ∷ []) "John.8.22"
∷ word (ἐ ∷ ∙λ ∷ θ ∷ ε ∷ ῖ ∷ ν ∷ []) "John.8.22"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.8.23"
∷ word (ἔ ∷ ∙λ ∷ ε ∷ γ ∷ ε ∷ ν ∷ []) "John.8.23"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.8.23"
∷ word (Ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.8.23"
∷ word (ἐ ∷ κ ∷ []) "John.8.23"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.8.23"
∷ word (κ ∷ ά ∷ τ ∷ ω ∷ []) "John.8.23"
∷ word (ἐ ∷ σ ∷ τ ∷ έ ∷ []) "John.8.23"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.8.23"
∷ word (ἐ ∷ κ ∷ []) "John.8.23"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.8.23"
∷ word (ἄ ∷ ν ∷ ω ∷ []) "John.8.23"
∷ word (ε ∷ ἰ ∷ μ ∷ ί ∷ []) "John.8.23"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.8.23"
∷ word (ἐ ∷ κ ∷ []) "John.8.23"
∷ word (τ ∷ ο ∷ ύ ∷ τ ∷ ο ∷ υ ∷ []) "John.8.23"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.8.23"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ υ ∷ []) "John.8.23"
∷ word (ἐ ∷ σ ∷ τ ∷ έ ∷ []) "John.8.23"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.8.23"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.8.23"
∷ word (ε ∷ ἰ ∷ μ ∷ ὶ ∷ []) "John.8.23"
∷ word (ἐ ∷ κ ∷ []) "John.8.23"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.8.23"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ υ ∷ []) "John.8.23"
∷ word (τ ∷ ο ∷ ύ ∷ τ ∷ ο ∷ υ ∷ []) "John.8.23"
∷ word (ε ∷ ἶ ∷ π ∷ ο ∷ ν ∷ []) "John.8.24"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.8.24"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.8.24"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.8.24"
∷ word (ἀ ∷ π ∷ ο ∷ θ ∷ α ∷ ν ∷ ε ∷ ῖ ∷ σ ∷ θ ∷ ε ∷ []) "John.8.24"
∷ word (ἐ ∷ ν ∷ []) "John.8.24"
∷ word (τ ∷ α ∷ ῖ ∷ ς ∷ []) "John.8.24"
∷ word (ἁ ∷ μ ∷ α ∷ ρ ∷ τ ∷ ί ∷ α ∷ ι ∷ ς ∷ []) "John.8.24"
∷ word (ὑ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.8.24"
∷ word (ἐ ∷ ὰ ∷ ν ∷ []) "John.8.24"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.8.24"
∷ word (μ ∷ ὴ ∷ []) "John.8.24"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ σ ∷ η ∷ τ ∷ ε ∷ []) "John.8.24"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.8.24"
∷ word (ἐ ∷ γ ∷ ώ ∷ []) "John.8.24"
∷ word (ε ∷ ἰ ∷ μ ∷ ι ∷ []) "John.8.24"
∷ word (ἀ ∷ π ∷ ο ∷ θ ∷ α ∷ ν ∷ ε ∷ ῖ ∷ σ ∷ θ ∷ ε ∷ []) "John.8.24"
∷ word (ἐ ∷ ν ∷ []) "John.8.24"
∷ word (τ ∷ α ∷ ῖ ∷ ς ∷ []) "John.8.24"
∷ word (ἁ ∷ μ ∷ α ∷ ρ ∷ τ ∷ ί ∷ α ∷ ι ∷ ς ∷ []) "John.8.24"
∷ word (ὑ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.8.24"
∷ word (ἔ ∷ ∙λ ∷ ε ∷ γ ∷ ο ∷ ν ∷ []) "John.8.25"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.8.25"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.8.25"
∷ word (Σ ∷ ὺ ∷ []) "John.8.25"
∷ word (τ ∷ ί ∷ ς ∷ []) "John.8.25"
∷ word (ε ∷ ἶ ∷ []) "John.8.25"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.8.25"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.8.25"
∷ word (ὁ ∷ []) "John.8.25"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.8.25"
∷ word (Τ ∷ ὴ ∷ ν ∷ []) "John.8.25"
∷ word (ἀ ∷ ρ ∷ χ ∷ ὴ ∷ ν ∷ []) "John.8.25"
∷ word (ὅ ∷ []) "John.8.25"
∷ word (τ ∷ ι ∷ []) "John.8.25"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.8.25"
∷ word (∙λ ∷ α ∷ ∙λ ∷ ῶ ∷ []) "John.8.25"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.8.25"
∷ word (π ∷ ο ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.8.26"
∷ word (ἔ ∷ χ ∷ ω ∷ []) "John.8.26"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.8.26"
∷ word (ὑ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.8.26"
∷ word (∙λ ∷ α ∷ ∙λ ∷ ε ∷ ῖ ∷ ν ∷ []) "John.8.26"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.8.26"
∷ word (κ ∷ ρ ∷ ί ∷ ν ∷ ε ∷ ι ∷ ν ∷ []) "John.8.26"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ []) "John.8.26"
∷ word (ὁ ∷ []) "John.8.26"
∷ word (π ∷ έ ∷ μ ∷ ψ ∷ α ∷ ς ∷ []) "John.8.26"
∷ word (μ ∷ ε ∷ []) "John.8.26"
∷ word (ἀ ∷ ∙λ ∷ η ∷ θ ∷ ή ∷ ς ∷ []) "John.8.26"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.8.26"
∷ word (κ ∷ ἀ ∷ γ ∷ ὼ ∷ []) "John.8.26"
∷ word (ἃ ∷ []) "John.8.26"
∷ word (ἤ ∷ κ ∷ ο ∷ υ ∷ σ ∷ α ∷ []) "John.8.26"
∷ word (π ∷ α ∷ ρ ∷ []) "John.8.26"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.8.26"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.8.26"
∷ word (∙λ ∷ α ∷ ∙λ ∷ ῶ ∷ []) "John.8.26"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.8.26"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.8.26"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ ν ∷ []) "John.8.26"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.8.27"
∷ word (ἔ ∷ γ ∷ ν ∷ ω ∷ σ ∷ α ∷ ν ∷ []) "John.8.27"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.8.27"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.8.27"
∷ word (π ∷ α ∷ τ ∷ έ ∷ ρ ∷ α ∷ []) "John.8.27"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.8.27"
∷ word (ἔ ∷ ∙λ ∷ ε ∷ γ ∷ ε ∷ ν ∷ []) "John.8.27"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.8.28"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.8.28"
∷ word (ὁ ∷ []) "John.8.28"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.8.28"
∷ word (Ὅ ∷ τ ∷ α ∷ ν ∷ []) "John.8.28"
∷ word (ὑ ∷ ψ ∷ ώ ∷ σ ∷ η ∷ τ ∷ ε ∷ []) "John.8.28"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.8.28"
∷ word (υ ∷ ἱ ∷ ὸ ∷ ν ∷ []) "John.8.28"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.8.28"
∷ word (ἀ ∷ ν ∷ θ ∷ ρ ∷ ώ ∷ π ∷ ο ∷ υ ∷ []) "John.8.28"
∷ word (τ ∷ ό ∷ τ ∷ ε ∷ []) "John.8.28"
∷ word (γ ∷ ν ∷ ώ ∷ σ ∷ ε ∷ σ ∷ θ ∷ ε ∷ []) "John.8.28"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.8.28"
∷ word (ἐ ∷ γ ∷ ώ ∷ []) "John.8.28"
∷ word (ε ∷ ἰ ∷ μ ∷ ι ∷ []) "John.8.28"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.8.28"
∷ word (ἀ ∷ π ∷ []) "John.8.28"
∷ word (ἐ ∷ μ ∷ α ∷ υ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.8.28"
∷ word (π ∷ ο ∷ ι ∷ ῶ ∷ []) "John.8.28"
∷ word (ο ∷ ὐ ∷ δ ∷ έ ∷ ν ∷ []) "John.8.28"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.8.28"
∷ word (κ ∷ α ∷ θ ∷ ὼ ∷ ς ∷ []) "John.8.28"
∷ word (ἐ ∷ δ ∷ ί ∷ δ ∷ α ∷ ξ ∷ έ ∷ ν ∷ []) "John.8.28"
∷ word (μ ∷ ε ∷ []) "John.8.28"
∷ word (ὁ ∷ []) "John.8.28"
∷ word (π ∷ α ∷ τ ∷ ὴ ∷ ρ ∷ []) "John.8.28"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.8.28"
∷ word (∙λ ∷ α ∷ ∙λ ∷ ῶ ∷ []) "John.8.28"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.8.29"
∷ word (ὁ ∷ []) "John.8.29"
∷ word (π ∷ έ ∷ μ ∷ ψ ∷ α ∷ ς ∷ []) "John.8.29"
∷ word (μ ∷ ε ∷ []) "John.8.29"
∷ word (μ ∷ ε ∷ τ ∷ []) "John.8.29"
∷ word (ἐ ∷ μ ∷ ο ∷ ῦ ∷ []) "John.8.29"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.8.29"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.8.29"
∷ word (ἀ ∷ φ ∷ ῆ ∷ κ ∷ έ ∷ ν ∷ []) "John.8.29"
∷ word (μ ∷ ε ∷ []) "John.8.29"
∷ word (μ ∷ ό ∷ ν ∷ ο ∷ ν ∷ []) "John.8.29"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.8.29"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.8.29"
∷ word (τ ∷ ὰ ∷ []) "John.8.29"
∷ word (ἀ ∷ ρ ∷ ε ∷ σ ∷ τ ∷ ὰ ∷ []) "John.8.29"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.8.29"
∷ word (π ∷ ο ∷ ι ∷ ῶ ∷ []) "John.8.29"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ ο ∷ τ ∷ ε ∷ []) "John.8.29"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.8.30"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.8.30"
∷ word (∙λ ∷ α ∷ ∙λ ∷ ο ∷ ῦ ∷ ν ∷ τ ∷ ο ∷ ς ∷ []) "John.8.30"
∷ word (π ∷ ο ∷ ∙λ ∷ ∙λ ∷ ο ∷ ὶ ∷ []) "John.8.30"
∷ word (ἐ ∷ π ∷ ί ∷ σ ∷ τ ∷ ε ∷ υ ∷ σ ∷ α ∷ ν ∷ []) "John.8.30"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.8.30"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.8.30"
∷ word (Ἔ ∷ ∙λ ∷ ε ∷ γ ∷ ε ∷ ν ∷ []) "John.8.31"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.8.31"
∷ word (ὁ ∷ []) "John.8.31"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.8.31"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.8.31"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.8.31"
∷ word (π ∷ ε ∷ π ∷ ι ∷ σ ∷ τ ∷ ε ∷ υ ∷ κ ∷ ό ∷ τ ∷ α ∷ ς ∷ []) "John.8.31"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.8.31"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ί ∷ ο ∷ υ ∷ ς ∷ []) "John.8.31"
∷ word (Ἐ ∷ ὰ ∷ ν ∷ []) "John.8.31"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.8.31"
∷ word (μ ∷ ε ∷ ί ∷ ν ∷ η ∷ τ ∷ ε ∷ []) "John.8.31"
∷ word (ἐ ∷ ν ∷ []) "John.8.31"
∷ word (τ ∷ ῷ ∷ []) "John.8.31"
∷ word (∙λ ∷ ό ∷ γ ∷ ῳ ∷ []) "John.8.31"
∷ word (τ ∷ ῷ ∷ []) "John.8.31"
∷ word (ἐ ∷ μ ∷ ῷ ∷ []) "John.8.31"
∷ word (ἀ ∷ ∙λ ∷ η ∷ θ ∷ ῶ ∷ ς ∷ []) "John.8.31"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ α ∷ ί ∷ []) "John.8.31"
∷ word (μ ∷ ο ∷ ύ ∷ []) "John.8.31"
∷ word (ἐ ∷ σ ∷ τ ∷ ε ∷ []) "John.8.31"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.8.32"
∷ word (γ ∷ ν ∷ ώ ∷ σ ∷ ε ∷ σ ∷ θ ∷ ε ∷ []) "John.8.32"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.8.32"
∷ word (ἀ ∷ ∙λ ∷ ή ∷ θ ∷ ε ∷ ι ∷ α ∷ ν ∷ []) "John.8.32"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.8.32"
∷ word (ἡ ∷ []) "John.8.32"
∷ word (ἀ ∷ ∙λ ∷ ή ∷ θ ∷ ε ∷ ι ∷ α ∷ []) "John.8.32"
∷ word (ἐ ∷ ∙λ ∷ ε ∷ υ ∷ θ ∷ ε ∷ ρ ∷ ώ ∷ σ ∷ ε ∷ ι ∷ []) "John.8.32"
∷ word (ὑ ∷ μ ∷ ᾶ ∷ ς ∷ []) "John.8.32"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.8.33"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.8.33"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.8.33"
∷ word (Σ ∷ π ∷ έ ∷ ρ ∷ μ ∷ α ∷ []) "John.8.33"
∷ word (Ἀ ∷ β ∷ ρ ∷ α ∷ ά ∷ μ ∷ []) "John.8.33"
∷ word (ἐ ∷ σ ∷ μ ∷ ε ∷ ν ∷ []) "John.8.33"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.8.33"
∷ word (ο ∷ ὐ ∷ δ ∷ ε ∷ ν ∷ ὶ ∷ []) "John.8.33"
∷ word (δ ∷ ε ∷ δ ∷ ο ∷ υ ∷ ∙λ ∷ ε ∷ ύ ∷ κ ∷ α ∷ μ ∷ ε ∷ ν ∷ []) "John.8.33"
∷ word (π ∷ ώ ∷ π ∷ ο ∷ τ ∷ ε ∷ []) "John.8.33"
∷ word (π ∷ ῶ ∷ ς ∷ []) "John.8.33"
∷ word (σ ∷ ὺ ∷ []) "John.8.33"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ ς ∷ []) "John.8.33"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.8.33"
∷ word (Ἐ ∷ ∙λ ∷ ε ∷ ύ ∷ θ ∷ ε ∷ ρ ∷ ο ∷ ι ∷ []) "John.8.33"
∷ word (γ ∷ ε ∷ ν ∷ ή ∷ σ ∷ ε ∷ σ ∷ θ ∷ ε ∷ []) "John.8.33"
∷ word (Ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.8.34"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.8.34"
∷ word (ὁ ∷ []) "John.8.34"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.8.34"
∷ word (Ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.8.34"
∷ word (ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.8.34"
∷ word (∙λ ∷ έ ∷ γ ∷ ω ∷ []) "John.8.34"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.8.34"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.8.34"
∷ word (π ∷ ᾶ ∷ ς ∷ []) "John.8.34"
∷ word (ὁ ∷ []) "John.8.34"
∷ word (π ∷ ο ∷ ι ∷ ῶ ∷ ν ∷ []) "John.8.34"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.8.34"
∷ word (ἁ ∷ μ ∷ α ∷ ρ ∷ τ ∷ ί ∷ α ∷ ν ∷ []) "John.8.34"
∷ word (δ ∷ ο ∷ ῦ ∷ ∙λ ∷ ό ∷ ς ∷ []) "John.8.34"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.8.34"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.8.34"
∷ word (ἁ ∷ μ ∷ α ∷ ρ ∷ τ ∷ ί ∷ α ∷ ς ∷ []) "John.8.34"
∷ word (ὁ ∷ []) "John.8.35"
∷ word (δ ∷ ὲ ∷ []) "John.8.35"
∷ word (δ ∷ ο ∷ ῦ ∷ ∙λ ∷ ο ∷ ς ∷ []) "John.8.35"
∷ word (ο ∷ ὐ ∷ []) "John.8.35"
∷ word (μ ∷ έ ∷ ν ∷ ε ∷ ι ∷ []) "John.8.35"
∷ word (ἐ ∷ ν ∷ []) "John.8.35"
∷ word (τ ∷ ῇ ∷ []) "John.8.35"
∷ word (ο ∷ ἰ ∷ κ ∷ ί ∷ ᾳ ∷ []) "John.8.35"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.8.35"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.8.35"
∷ word (α ∷ ἰ ∷ ῶ ∷ ν ∷ α ∷ []) "John.8.35"
∷ word (ὁ ∷ []) "John.8.35"
∷ word (υ ∷ ἱ ∷ ὸ ∷ ς ∷ []) "John.8.35"
∷ word (μ ∷ έ ∷ ν ∷ ε ∷ ι ∷ []) "John.8.35"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.8.35"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.8.35"
∷ word (α ∷ ἰ ∷ ῶ ∷ ν ∷ α ∷ []) "John.8.35"
∷ word (ἐ ∷ ὰ ∷ ν ∷ []) "John.8.36"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.8.36"
∷ word (ὁ ∷ []) "John.8.36"
∷ word (υ ∷ ἱ ∷ ὸ ∷ ς ∷ []) "John.8.36"
∷ word (ὑ ∷ μ ∷ ᾶ ∷ ς ∷ []) "John.8.36"
∷ word (ἐ ∷ ∙λ ∷ ε ∷ υ ∷ θ ∷ ε ∷ ρ ∷ ώ ∷ σ ∷ ῃ ∷ []) "John.8.36"
∷ word (ὄ ∷ ν ∷ τ ∷ ω ∷ ς ∷ []) "John.8.36"
∷ word (ἐ ∷ ∙λ ∷ ε ∷ ύ ∷ θ ∷ ε ∷ ρ ∷ ο ∷ ι ∷ []) "John.8.36"
∷ word (ἔ ∷ σ ∷ ε ∷ σ ∷ θ ∷ ε ∷ []) "John.8.36"
∷ word (ο ∷ ἶ ∷ δ ∷ α ∷ []) "John.8.37"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.8.37"
∷ word (σ ∷ π ∷ έ ∷ ρ ∷ μ ∷ α ∷ []) "John.8.37"
∷ word (Ἀ ∷ β ∷ ρ ∷ α ∷ ά ∷ μ ∷ []) "John.8.37"
∷ word (ἐ ∷ σ ∷ τ ∷ ε ∷ []) "John.8.37"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.8.37"
∷ word (ζ ∷ η ∷ τ ∷ ε ∷ ῖ ∷ τ ∷ έ ∷ []) "John.8.37"
∷ word (μ ∷ ε ∷ []) "John.8.37"
∷ word (ἀ ∷ π ∷ ο ∷ κ ∷ τ ∷ ε ∷ ῖ ∷ ν ∷ α ∷ ι ∷ []) "John.8.37"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.8.37"
∷ word (ὁ ∷ []) "John.8.37"
∷ word (∙λ ∷ ό ∷ γ ∷ ο ∷ ς ∷ []) "John.8.37"
∷ word (ὁ ∷ []) "John.8.37"
∷ word (ἐ ∷ μ ∷ ὸ ∷ ς ∷ []) "John.8.37"
∷ word (ο ∷ ὐ ∷ []) "John.8.37"
∷ word (χ ∷ ω ∷ ρ ∷ ε ∷ ῖ ∷ []) "John.8.37"
∷ word (ἐ ∷ ν ∷ []) "John.8.37"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.8.37"
∷ word (ἃ ∷ []) "John.8.38"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.8.38"
∷ word (ἑ ∷ ώ ∷ ρ ∷ α ∷ κ ∷ α ∷ []) "John.8.38"
∷ word (π ∷ α ∷ ρ ∷ ὰ ∷ []) "John.8.38"
∷ word (τ ∷ ῷ ∷ []) "John.8.38"
∷ word (π ∷ α ∷ τ ∷ ρ ∷ ὶ ∷ []) "John.8.38"
∷ word (∙λ ∷ α ∷ ∙λ ∷ ῶ ∷ []) "John.8.38"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.8.38"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.8.38"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.8.38"
∷ word (ἃ ∷ []) "John.8.38"
∷ word (ἠ ∷ κ ∷ ο ∷ ύ ∷ σ ∷ α ∷ τ ∷ ε ∷ []) "John.8.38"
∷ word (π ∷ α ∷ ρ ∷ ὰ ∷ []) "John.8.38"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.8.38"
∷ word (π ∷ α ∷ τ ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.8.38"
∷ word (π ∷ ο ∷ ι ∷ ε ∷ ῖ ∷ τ ∷ ε ∷ []) "John.8.38"
∷ word (Ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.8.39"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.8.39"
∷ word (ε ∷ ἶ ∷ π ∷ α ∷ ν ∷ []) "John.8.39"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.8.39"
∷ word (Ὁ ∷ []) "John.8.39"
∷ word (π ∷ α ∷ τ ∷ ὴ ∷ ρ ∷ []) "John.8.39"
∷ word (ἡ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.8.39"
∷ word (Ἀ ∷ β ∷ ρ ∷ α ∷ ά ∷ μ ∷ []) "John.8.39"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.8.39"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.8.39"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.8.39"
∷ word (ὁ ∷ []) "John.8.39"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.8.39"
∷ word (Ε ∷ ἰ ∷ []) "John.8.39"
∷ word (τ ∷ έ ∷ κ ∷ ν ∷ α ∷ []) "John.8.39"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.8.39"
∷ word (Ἀ ∷ β ∷ ρ ∷ α ∷ ά ∷ μ ∷ []) "John.8.39"
∷ word (ἐ ∷ σ ∷ τ ∷ ε ∷ []) "John.8.39"
∷ word (τ ∷ ὰ ∷ []) "John.8.39"
∷ word (ἔ ∷ ρ ∷ γ ∷ α ∷ []) "John.8.39"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.8.39"
∷ word (Ἀ ∷ β ∷ ρ ∷ α ∷ ὰ ∷ μ ∷ []) "John.8.39"
∷ word (ἐ ∷ π ∷ ο ∷ ι ∷ ε ∷ ῖ ∷ τ ∷ ε ∷ []) "John.8.39"
∷ word (ν ∷ ῦ ∷ ν ∷ []) "John.8.40"
∷ word (δ ∷ ὲ ∷ []) "John.8.40"
∷ word (ζ ∷ η ∷ τ ∷ ε ∷ ῖ ∷ τ ∷ έ ∷ []) "John.8.40"
∷ word (μ ∷ ε ∷ []) "John.8.40"
∷ word (ἀ ∷ π ∷ ο ∷ κ ∷ τ ∷ ε ∷ ῖ ∷ ν ∷ α ∷ ι ∷ []) "John.8.40"
∷ word (ἄ ∷ ν ∷ θ ∷ ρ ∷ ω ∷ π ∷ ο ∷ ν ∷ []) "John.8.40"
∷ word (ὃ ∷ ς ∷ []) "John.8.40"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.8.40"
∷ word (ἀ ∷ ∙λ ∷ ή ∷ θ ∷ ε ∷ ι ∷ α ∷ ν ∷ []) "John.8.40"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.8.40"
∷ word (∙λ ∷ ε ∷ ∙λ ∷ ά ∷ ∙λ ∷ η ∷ κ ∷ α ∷ []) "John.8.40"
∷ word (ἣ ∷ ν ∷ []) "John.8.40"
∷ word (ἤ ∷ κ ∷ ο ∷ υ ∷ σ ∷ α ∷ []) "John.8.40"
∷ word (π ∷ α ∷ ρ ∷ ὰ ∷ []) "John.8.40"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.8.40"
∷ word (θ ∷ ε ∷ ο ∷ ῦ ∷ []) "John.8.40"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.8.40"
∷ word (Ἀ ∷ β ∷ ρ ∷ α ∷ ὰ ∷ μ ∷ []) "John.8.40"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.8.40"
∷ word (ἐ ∷ π ∷ ο ∷ ί ∷ η ∷ σ ∷ ε ∷ ν ∷ []) "John.8.40"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.8.41"
∷ word (π ∷ ο ∷ ι ∷ ε ∷ ῖ ∷ τ ∷ ε ∷ []) "John.8.41"
∷ word (τ ∷ ὰ ∷ []) "John.8.41"
∷ word (ἔ ∷ ρ ∷ γ ∷ α ∷ []) "John.8.41"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.8.41"
∷ word (π ∷ α ∷ τ ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.8.41"
∷ word (ὑ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.8.41"
∷ word (ε ∷ ἶ ∷ π ∷ α ∷ ν ∷ []) "John.8.41"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.8.41"
∷ word (Ἡ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.8.41"
∷ word (ἐ ∷ κ ∷ []) "John.8.41"
∷ word (π ∷ ο ∷ ρ ∷ ν ∷ ε ∷ ί ∷ α ∷ ς ∷ []) "John.8.41"
∷ word (ο ∷ ὐ ∷ []) "John.8.41"
∷ word (γ ∷ ε ∷ γ ∷ ε ∷ ν ∷ ν ∷ ή ∷ μ ∷ ε ∷ θ ∷ α ∷ []) "John.8.41"
∷ word (ἕ ∷ ν ∷ α ∷ []) "John.8.41"
∷ word (π ∷ α ∷ τ ∷ έ ∷ ρ ∷ α ∷ []) "John.8.41"
∷ word (ἔ ∷ χ ∷ ο ∷ μ ∷ ε ∷ ν ∷ []) "John.8.41"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.8.41"
∷ word (θ ∷ ε ∷ ό ∷ ν ∷ []) "John.8.41"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.8.42"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.8.42"
∷ word (ὁ ∷ []) "John.8.42"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.8.42"
∷ word (Ε ∷ ἰ ∷ []) "John.8.42"
∷ word (ὁ ∷ []) "John.8.42"
∷ word (θ ∷ ε ∷ ὸ ∷ ς ∷ []) "John.8.42"
∷ word (π ∷ α ∷ τ ∷ ὴ ∷ ρ ∷ []) "John.8.42"
∷ word (ὑ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.8.42"
∷ word (ἦ ∷ ν ∷ []) "John.8.42"
∷ word (ἠ ∷ γ ∷ α ∷ π ∷ ᾶ ∷ τ ∷ ε ∷ []) "John.8.42"
∷ word (ἂ ∷ ν ∷ []) "John.8.42"
∷ word (ἐ ∷ μ ∷ έ ∷ []) "John.8.42"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.8.42"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.8.42"
∷ word (ἐ ∷ κ ∷ []) "John.8.42"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.8.42"
∷ word (θ ∷ ε ∷ ο ∷ ῦ ∷ []) "John.8.42"
∷ word (ἐ ∷ ξ ∷ ῆ ∷ ∙λ ∷ θ ∷ ο ∷ ν ∷ []) "John.8.42"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.8.42"
∷ word (ἥ ∷ κ ∷ ω ∷ []) "John.8.42"
∷ word (ο ∷ ὐ ∷ δ ∷ ὲ ∷ []) "John.8.42"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.8.42"
∷ word (ἀ ∷ π ∷ []) "John.8.42"
∷ word (ἐ ∷ μ ∷ α ∷ υ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.8.42"
∷ word (ἐ ∷ ∙λ ∷ ή ∷ ∙λ ∷ υ ∷ θ ∷ α ∷ []) "John.8.42"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ []) "John.8.42"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ό ∷ ς ∷ []) "John.8.42"
∷ word (μ ∷ ε ∷ []) "John.8.42"
∷ word (ἀ ∷ π ∷ έ ∷ σ ∷ τ ∷ ε ∷ ι ∷ ∙λ ∷ ε ∷ ν ∷ []) "John.8.42"
∷ word (δ ∷ ι ∷ ὰ ∷ []) "John.8.43"
∷ word (τ ∷ ί ∷ []) "John.8.43"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.8.43"
∷ word (∙λ ∷ α ∷ ∙λ ∷ ι ∷ ὰ ∷ ν ∷ []) "John.8.43"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.8.43"
∷ word (ἐ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.8.43"
∷ word (ο ∷ ὐ ∷ []) "John.8.43"
∷ word (γ ∷ ι ∷ ν ∷ ώ ∷ σ ∷ κ ∷ ε ∷ τ ∷ ε ∷ []) "John.8.43"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.8.43"
∷ word (ο ∷ ὐ ∷ []) "John.8.43"
∷ word (δ ∷ ύ ∷ ν ∷ α ∷ σ ∷ θ ∷ ε ∷ []) "John.8.43"
∷ word (ἀ ∷ κ ∷ ο ∷ ύ ∷ ε ∷ ι ∷ ν ∷ []) "John.8.43"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.8.43"
∷ word (∙λ ∷ ό ∷ γ ∷ ο ∷ ν ∷ []) "John.8.43"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.8.43"
∷ word (ἐ ∷ μ ∷ ό ∷ ν ∷ []) "John.8.43"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.8.44"
∷ word (ἐ ∷ κ ∷ []) "John.8.44"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.8.44"
∷ word (π ∷ α ∷ τ ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.8.44"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.8.44"
∷ word (δ ∷ ι ∷ α ∷ β ∷ ό ∷ ∙λ ∷ ο ∷ υ ∷ []) "John.8.44"
∷ word (ἐ ∷ σ ∷ τ ∷ ὲ ∷ []) "John.8.44"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.8.44"
∷ word (τ ∷ ὰ ∷ ς ∷ []) "John.8.44"
∷ word (ἐ ∷ π ∷ ι ∷ θ ∷ υ ∷ μ ∷ ί ∷ α ∷ ς ∷ []) "John.8.44"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.8.44"
∷ word (π ∷ α ∷ τ ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.8.44"
∷ word (ὑ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.8.44"
∷ word (θ ∷ έ ∷ ∙λ ∷ ε ∷ τ ∷ ε ∷ []) "John.8.44"
∷ word (π ∷ ο ∷ ι ∷ ε ∷ ῖ ∷ ν ∷ []) "John.8.44"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ο ∷ ς ∷ []) "John.8.44"
∷ word (ἀ ∷ ν ∷ θ ∷ ρ ∷ ω ∷ π ∷ ο ∷ κ ∷ τ ∷ ό ∷ ν ∷ ο ∷ ς ∷ []) "John.8.44"
∷ word (ἦ ∷ ν ∷ []) "John.8.44"
∷ word (ἀ ∷ π ∷ []) "John.8.44"
∷ word (ἀ ∷ ρ ∷ χ ∷ ῆ ∷ ς ∷ []) "John.8.44"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.8.44"
∷ word (ἐ ∷ ν ∷ []) "John.8.44"
∷ word (τ ∷ ῇ ∷ []) "John.8.44"
∷ word (ἀ ∷ ∙λ ∷ η ∷ θ ∷ ε ∷ ί ∷ ᾳ ∷ []) "John.8.44"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.8.44"
∷ word (ἔ ∷ σ ∷ τ ∷ η ∷ κ ∷ ε ∷ ν ∷ []) "John.8.44"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.8.44"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.8.44"
∷ word (ἔ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.8.44"
∷ word (ἀ ∷ ∙λ ∷ ή ∷ θ ∷ ε ∷ ι ∷ α ∷ []) "John.8.44"
∷ word (ἐ ∷ ν ∷ []) "John.8.44"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.8.44"
∷ word (ὅ ∷ τ ∷ α ∷ ν ∷ []) "John.8.44"
∷ word (∙λ ∷ α ∷ ∙λ ∷ ῇ ∷ []) "John.8.44"
∷ word (τ ∷ ὸ ∷ []) "John.8.44"
∷ word (ψ ∷ ε ∷ ῦ ∷ δ ∷ ο ∷ ς ∷ []) "John.8.44"
∷ word (ἐ ∷ κ ∷ []) "John.8.44"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.8.44"
∷ word (ἰ ∷ δ ∷ ί ∷ ω ∷ ν ∷ []) "John.8.44"
∷ word (∙λ ∷ α ∷ ∙λ ∷ ε ∷ ῖ ∷ []) "John.8.44"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.8.44"
∷ word (ψ ∷ ε ∷ ύ ∷ σ ∷ τ ∷ η ∷ ς ∷ []) "John.8.44"
∷ word (ἐ ∷ σ ∷ τ ∷ ὶ ∷ ν ∷ []) "John.8.44"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.8.44"
∷ word (ὁ ∷ []) "John.8.44"
∷ word (π ∷ α ∷ τ ∷ ὴ ∷ ρ ∷ []) "John.8.44"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.8.44"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.8.45"
∷ word (δ ∷ ὲ ∷ []) "John.8.45"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.8.45"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.8.45"
∷ word (ἀ ∷ ∙λ ∷ ή ∷ θ ∷ ε ∷ ι ∷ α ∷ ν ∷ []) "John.8.45"
∷ word (∙λ ∷ έ ∷ γ ∷ ω ∷ []) "John.8.45"
∷ word (ο ∷ ὐ ∷ []) "John.8.45"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ ε ∷ τ ∷ έ ∷ []) "John.8.45"
∷ word (μ ∷ ο ∷ ι ∷ []) "John.8.45"
∷ word (τ ∷ ί ∷ ς ∷ []) "John.8.46"
∷ word (ἐ ∷ ξ ∷ []) "John.8.46"
∷ word (ὑ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.8.46"
∷ word (ἐ ∷ ∙λ ∷ έ ∷ γ ∷ χ ∷ ε ∷ ι ∷ []) "John.8.46"
∷ word (μ ∷ ε ∷ []) "John.8.46"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.8.46"
∷ word (ἁ ∷ μ ∷ α ∷ ρ ∷ τ ∷ ί ∷ α ∷ ς ∷ []) "John.8.46"
∷ word (ε ∷ ἰ ∷ []) "John.8.46"
∷ word (ἀ ∷ ∙λ ∷ ή ∷ θ ∷ ε ∷ ι ∷ α ∷ ν ∷ []) "John.8.46"
∷ word (∙λ ∷ έ ∷ γ ∷ ω ∷ []) "John.8.46"
∷ word (δ ∷ ι ∷ ὰ ∷ []) "John.8.46"
∷ word (τ ∷ ί ∷ []) "John.8.46"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.8.46"
∷ word (ο ∷ ὐ ∷ []) "John.8.46"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ ε ∷ τ ∷ έ ∷ []) "John.8.46"
∷ word (μ ∷ ο ∷ ι ∷ []) "John.8.46"
∷ word (ὁ ∷ []) "John.8.47"
∷ word (ὢ ∷ ν ∷ []) "John.8.47"
∷ word (ἐ ∷ κ ∷ []) "John.8.47"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.8.47"
∷ word (θ ∷ ε ∷ ο ∷ ῦ ∷ []) "John.8.47"
∷ word (τ ∷ ὰ ∷ []) "John.8.47"
∷ word (ῥ ∷ ή ∷ μ ∷ α ∷ τ ∷ α ∷ []) "John.8.47"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.8.47"
∷ word (θ ∷ ε ∷ ο ∷ ῦ ∷ []) "John.8.47"
∷ word (ἀ ∷ κ ∷ ο ∷ ύ ∷ ε ∷ ι ∷ []) "John.8.47"
∷ word (δ ∷ ι ∷ ὰ ∷ []) "John.8.47"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.8.47"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.8.47"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.8.47"
∷ word (ἀ ∷ κ ∷ ο ∷ ύ ∷ ε ∷ τ ∷ ε ∷ []) "John.8.47"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.8.47"
∷ word (ἐ ∷ κ ∷ []) "John.8.47"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.8.47"
∷ word (θ ∷ ε ∷ ο ∷ ῦ ∷ []) "John.8.47"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.8.47"
∷ word (ἐ ∷ σ ∷ τ ∷ έ ∷ []) "John.8.47"
∷ word (Ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.8.48"
∷ word (ο ∷ ἱ ∷ []) "John.8.48"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ῖ ∷ ο ∷ ι ∷ []) "John.8.48"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.8.48"
∷ word (ε ∷ ἶ ∷ π ∷ α ∷ ν ∷ []) "John.8.48"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.8.48"
∷ word (Ο ∷ ὐ ∷ []) "John.8.48"
∷ word (κ ∷ α ∷ ∙λ ∷ ῶ ∷ ς ∷ []) "John.8.48"
∷ word (∙λ ∷ έ ∷ γ ∷ ο ∷ μ ∷ ε ∷ ν ∷ []) "John.8.48"
∷ word (ἡ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.8.48"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.8.48"
∷ word (Σ ∷ α ∷ μ ∷ α ∷ ρ ∷ ί ∷ τ ∷ η ∷ ς ∷ []) "John.8.48"
∷ word (ε ∷ ἶ ∷ []) "John.8.48"
∷ word (σ ∷ ὺ ∷ []) "John.8.48"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.8.48"
∷ word (δ ∷ α ∷ ι ∷ μ ∷ ό ∷ ν ∷ ι ∷ ο ∷ ν ∷ []) "John.8.48"
∷ word (ἔ ∷ χ ∷ ε ∷ ι ∷ ς ∷ []) "John.8.48"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.8.49"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.8.49"
∷ word (Ἐ ∷ γ ∷ ὼ ∷ []) "John.8.49"
∷ word (δ ∷ α ∷ ι ∷ μ ∷ ό ∷ ν ∷ ι ∷ ο ∷ ν ∷ []) "John.8.49"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.8.49"
∷ word (ἔ ∷ χ ∷ ω ∷ []) "John.8.49"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.8.49"
∷ word (τ ∷ ι ∷ μ ∷ ῶ ∷ []) "John.8.49"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.8.49"
∷ word (π ∷ α ∷ τ ∷ έ ∷ ρ ∷ α ∷ []) "John.8.49"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.8.49"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.8.49"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.8.49"
∷ word (ἀ ∷ τ ∷ ι ∷ μ ∷ ά ∷ ζ ∷ ε ∷ τ ∷ έ ∷ []) "John.8.49"
∷ word (μ ∷ ε ∷ []) "John.8.49"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.8.50"
∷ word (δ ∷ ὲ ∷ []) "John.8.50"
∷ word (ο ∷ ὐ ∷ []) "John.8.50"
∷ word (ζ ∷ η ∷ τ ∷ ῶ ∷ []) "John.8.50"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.8.50"
∷ word (δ ∷ ό ∷ ξ ∷ α ∷ ν ∷ []) "John.8.50"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.8.50"
∷ word (ἔ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.8.50"
∷ word (ὁ ∷ []) "John.8.50"
∷ word (ζ ∷ η ∷ τ ∷ ῶ ∷ ν ∷ []) "John.8.50"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.8.50"
∷ word (κ ∷ ρ ∷ ί ∷ ν ∷ ω ∷ ν ∷ []) "John.8.50"
∷ word (ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.8.51"
∷ word (ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.8.51"
∷ word (∙λ ∷ έ ∷ γ ∷ ω ∷ []) "John.8.51"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.8.51"
∷ word (ἐ ∷ ά ∷ ν ∷ []) "John.8.51"
∷ word (τ ∷ ι ∷ ς ∷ []) "John.8.51"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.8.51"
∷ word (ἐ ∷ μ ∷ ὸ ∷ ν ∷ []) "John.8.51"
∷ word (∙λ ∷ ό ∷ γ ∷ ο ∷ ν ∷ []) "John.8.51"
∷ word (τ ∷ η ∷ ρ ∷ ή ∷ σ ∷ ῃ ∷ []) "John.8.51"
∷ word (θ ∷ ά ∷ ν ∷ α ∷ τ ∷ ο ∷ ν ∷ []) "John.8.51"
∷ word (ο ∷ ὐ ∷ []) "John.8.51"
∷ word (μ ∷ ὴ ∷ []) "John.8.51"
∷ word (θ ∷ ε ∷ ω ∷ ρ ∷ ή ∷ σ ∷ ῃ ∷ []) "John.8.51"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.8.51"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.8.51"
∷ word (α ∷ ἰ ∷ ῶ ∷ ν ∷ α ∷ []) "John.8.51"
∷ word (ε ∷ ἶ ∷ π ∷ ο ∷ ν ∷ []) "John.8.52"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.8.52"
∷ word (ο ∷ ἱ ∷ []) "John.8.52"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ῖ ∷ ο ∷ ι ∷ []) "John.8.52"
∷ word (Ν ∷ ῦ ∷ ν ∷ []) "John.8.52"
∷ word (ἐ ∷ γ ∷ ν ∷ ώ ∷ κ ∷ α ∷ μ ∷ ε ∷ ν ∷ []) "John.8.52"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.8.52"
∷ word (δ ∷ α ∷ ι ∷ μ ∷ ό ∷ ν ∷ ι ∷ ο ∷ ν ∷ []) "John.8.52"
∷ word (ἔ ∷ χ ∷ ε ∷ ι ∷ ς ∷ []) "John.8.52"
∷ word (Ἀ ∷ β ∷ ρ ∷ α ∷ ὰ ∷ μ ∷ []) "John.8.52"
∷ word (ἀ ∷ π ∷ έ ∷ θ ∷ α ∷ ν ∷ ε ∷ ν ∷ []) "John.8.52"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.8.52"
∷ word (ο ∷ ἱ ∷ []) "John.8.52"
∷ word (π ∷ ρ ∷ ο ∷ φ ∷ ῆ ∷ τ ∷ α ∷ ι ∷ []) "John.8.52"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.8.52"
∷ word (σ ∷ ὺ ∷ []) "John.8.52"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ ς ∷ []) "John.8.52"
∷ word (Ἐ ∷ ά ∷ ν ∷ []) "John.8.52"
∷ word (τ ∷ ι ∷ ς ∷ []) "John.8.52"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.8.52"
∷ word (∙λ ∷ ό ∷ γ ∷ ο ∷ ν ∷ []) "John.8.52"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.8.52"
∷ word (τ ∷ η ∷ ρ ∷ ή ∷ σ ∷ ῃ ∷ []) "John.8.52"
∷ word (ο ∷ ὐ ∷ []) "John.8.52"
∷ word (μ ∷ ὴ ∷ []) "John.8.52"
∷ word (γ ∷ ε ∷ ύ ∷ σ ∷ η ∷ τ ∷ α ∷ ι ∷ []) "John.8.52"
∷ word (θ ∷ α ∷ ν ∷ ά ∷ τ ∷ ο ∷ υ ∷ []) "John.8.52"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.8.52"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.8.52"
∷ word (α ∷ ἰ ∷ ῶ ∷ ν ∷ α ∷ []) "John.8.52"
∷ word (μ ∷ ὴ ∷ []) "John.8.53"
∷ word (σ ∷ ὺ ∷ []) "John.8.53"
∷ word (μ ∷ ε ∷ ί ∷ ζ ∷ ω ∷ ν ∷ []) "John.8.53"
∷ word (ε ∷ ἶ ∷ []) "John.8.53"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.8.53"
∷ word (π ∷ α ∷ τ ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.8.53"
∷ word (ἡ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.8.53"
∷ word (Ἀ ∷ β ∷ ρ ∷ α ∷ ά ∷ μ ∷ []) "John.8.53"
∷ word (ὅ ∷ σ ∷ τ ∷ ι ∷ ς ∷ []) "John.8.53"
∷ word (ἀ ∷ π ∷ έ ∷ θ ∷ α ∷ ν ∷ ε ∷ ν ∷ []) "John.8.53"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.8.53"
∷ word (ο ∷ ἱ ∷ []) "John.8.53"
∷ word (π ∷ ρ ∷ ο ∷ φ ∷ ῆ ∷ τ ∷ α ∷ ι ∷ []) "John.8.53"
∷ word (ἀ ∷ π ∷ έ ∷ θ ∷ α ∷ ν ∷ ο ∷ ν ∷ []) "John.8.53"
∷ word (τ ∷ ί ∷ ν ∷ α ∷ []) "John.8.53"
∷ word (σ ∷ ε ∷ α ∷ υ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.8.53"
∷ word (π ∷ ο ∷ ι ∷ ε ∷ ῖ ∷ ς ∷ []) "John.8.53"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.8.54"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.8.54"
∷ word (Ἐ ∷ ὰ ∷ ν ∷ []) "John.8.54"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.8.54"
∷ word (δ ∷ ο ∷ ξ ∷ ά ∷ σ ∷ ω ∷ []) "John.8.54"
∷ word (ἐ ∷ μ ∷ α ∷ υ ∷ τ ∷ ό ∷ ν ∷ []) "John.8.54"
∷ word (ἡ ∷ []) "John.8.54"
∷ word (δ ∷ ό ∷ ξ ∷ α ∷ []) "John.8.54"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.8.54"
∷ word (ο ∷ ὐ ∷ δ ∷ έ ∷ ν ∷ []) "John.8.54"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.8.54"
∷ word (ἔ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.8.54"
∷ word (ὁ ∷ []) "John.8.54"
∷ word (π ∷ α ∷ τ ∷ ή ∷ ρ ∷ []) "John.8.54"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.8.54"
∷ word (ὁ ∷ []) "John.8.54"
∷ word (δ ∷ ο ∷ ξ ∷ ά ∷ ζ ∷ ω ∷ ν ∷ []) "John.8.54"
∷ word (μ ∷ ε ∷ []) "John.8.54"
∷ word (ὃ ∷ ν ∷ []) "John.8.54"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.8.54"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ τ ∷ ε ∷ []) "John.8.54"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.8.54"
∷ word (θ ∷ ε ∷ ὸ ∷ ς ∷ []) "John.8.54"
∷ word (ἡ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.8.54"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.8.54"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.8.55"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.8.55"
∷ word (ἐ ∷ γ ∷ ν ∷ ώ ∷ κ ∷ α ∷ τ ∷ ε ∷ []) "John.8.55"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.8.55"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.8.55"
∷ word (δ ∷ ὲ ∷ []) "John.8.55"
∷ word (ο ∷ ἶ ∷ δ ∷ α ∷ []) "John.8.55"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.8.55"
∷ word (κ ∷ ἂ ∷ ν ∷ []) "John.8.55"
∷ word (ε ∷ ἴ ∷ π ∷ ω ∷ []) "John.8.55"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.8.55"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.8.55"
∷ word (ο ∷ ἶ ∷ δ ∷ α ∷ []) "John.8.55"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.8.55"
∷ word (ἔ ∷ σ ∷ ο ∷ μ ∷ α ∷ ι ∷ []) "John.8.55"
∷ word (ὅ ∷ μ ∷ ο ∷ ι ∷ ο ∷ ς ∷ []) "John.8.55"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.8.55"
∷ word (ψ ∷ ε ∷ ύ ∷ σ ∷ τ ∷ η ∷ ς ∷ []) "John.8.55"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.8.55"
∷ word (ο ∷ ἶ ∷ δ ∷ α ∷ []) "John.8.55"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.8.55"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.8.55"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.8.55"
∷ word (∙λ ∷ ό ∷ γ ∷ ο ∷ ν ∷ []) "John.8.55"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.8.55"
∷ word (τ ∷ η ∷ ρ ∷ ῶ ∷ []) "John.8.55"
∷ word (Ἀ ∷ β ∷ ρ ∷ α ∷ ὰ ∷ μ ∷ []) "John.8.56"
∷ word (ὁ ∷ []) "John.8.56"
∷ word (π ∷ α ∷ τ ∷ ὴ ∷ ρ ∷ []) "John.8.56"
∷ word (ὑ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.8.56"
∷ word (ἠ ∷ γ ∷ α ∷ ∙λ ∷ ∙λ ∷ ι ∷ ά ∷ σ ∷ α ∷ τ ∷ ο ∷ []) "John.8.56"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.8.56"
∷ word (ἴ ∷ δ ∷ ῃ ∷ []) "John.8.56"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.8.56"
∷ word (ἡ ∷ μ ∷ έ ∷ ρ ∷ α ∷ ν ∷ []) "John.8.56"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.8.56"
∷ word (ἐ ∷ μ ∷ ή ∷ ν ∷ []) "John.8.56"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.8.56"
∷ word (ε ∷ ἶ ∷ δ ∷ ε ∷ ν ∷ []) "John.8.56"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.8.56"
∷ word (ἐ ∷ χ ∷ ά ∷ ρ ∷ η ∷ []) "John.8.56"
∷ word (ε ∷ ἶ ∷ π ∷ ο ∷ ν ∷ []) "John.8.57"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.8.57"
∷ word (ο ∷ ἱ ∷ []) "John.8.57"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ῖ ∷ ο ∷ ι ∷ []) "John.8.57"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.8.57"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.8.57"
∷ word (Π ∷ ε ∷ ν ∷ τ ∷ ή ∷ κ ∷ ο ∷ ν ∷ τ ∷ α ∷ []) "John.8.57"
∷ word (ἔ ∷ τ ∷ η ∷ []) "John.8.57"
∷ word (ο ∷ ὔ ∷ π ∷ ω ∷ []) "John.8.57"
∷ word (ἔ ∷ χ ∷ ε ∷ ι ∷ ς ∷ []) "John.8.57"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.8.57"
∷ word (Ἀ ∷ β ∷ ρ ∷ α ∷ ὰ ∷ μ ∷ []) "John.8.57"
∷ word (ἑ ∷ ώ ∷ ρ ∷ α ∷ κ ∷ α ∷ ς ∷ []) "John.8.57"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.8.58"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.8.58"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.8.58"
∷ word (Ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.8.58"
∷ word (ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.8.58"
∷ word (∙λ ∷ έ ∷ γ ∷ ω ∷ []) "John.8.58"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.8.58"
∷ word (π ∷ ρ ∷ ὶ ∷ ν ∷ []) "John.8.58"
∷ word (Ἀ ∷ β ∷ ρ ∷ α ∷ ὰ ∷ μ ∷ []) "John.8.58"
∷ word (γ ∷ ε ∷ ν ∷ έ ∷ σ ∷ θ ∷ α ∷ ι ∷ []) "John.8.58"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.8.58"
∷ word (ε ∷ ἰ ∷ μ ∷ ί ∷ []) "John.8.58"
∷ word (ἦ ∷ ρ ∷ α ∷ ν ∷ []) "John.8.59"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.8.59"
∷ word (∙λ ∷ ί ∷ θ ∷ ο ∷ υ ∷ ς ∷ []) "John.8.59"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.8.59"
∷ word (β ∷ ά ∷ ∙λ ∷ ω ∷ σ ∷ ι ∷ ν ∷ []) "John.8.59"
∷ word (ἐ ∷ π ∷ []) "John.8.59"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.8.59"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.8.59"
∷ word (δ ∷ ὲ ∷ []) "John.8.59"
∷ word (ἐ ∷ κ ∷ ρ ∷ ύ ∷ β ∷ η ∷ []) "John.8.59"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.8.59"
∷ word (ἐ ∷ ξ ∷ ῆ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.8.59"
∷ word (ἐ ∷ κ ∷ []) "John.8.59"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.8.59"
∷ word (ἱ ∷ ε ∷ ρ ∷ ο ∷ ῦ ∷ []) "John.8.59"
∷ word (Κ ∷ α ∷ ὶ ∷ []) "John.9.1"
∷ word (π ∷ α ∷ ρ ∷ ά ∷ γ ∷ ω ∷ ν ∷ []) "John.9.1"
∷ word (ε ∷ ἶ ∷ δ ∷ ε ∷ ν ∷ []) "John.9.1"
∷ word (ἄ ∷ ν ∷ θ ∷ ρ ∷ ω ∷ π ∷ ο ∷ ν ∷ []) "John.9.1"
∷ word (τ ∷ υ ∷ φ ∷ ∙λ ∷ ὸ ∷ ν ∷ []) "John.9.1"
∷ word (ἐ ∷ κ ∷ []) "John.9.1"
∷ word (γ ∷ ε ∷ ν ∷ ε ∷ τ ∷ ῆ ∷ ς ∷ []) "John.9.1"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.9.2"
∷ word (ἠ ∷ ρ ∷ ώ ∷ τ ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.9.2"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.9.2"
∷ word (ο ∷ ἱ ∷ []) "John.9.2"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ α ∷ ὶ ∷ []) "John.9.2"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.9.2"
∷ word (∙λ ∷ έ ∷ γ ∷ ο ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.9.2"
∷ word (Ῥ ∷ α ∷ β ∷ β ∷ ί ∷ []) "John.9.2"
∷ word (τ ∷ ί ∷ ς ∷ []) "John.9.2"
∷ word (ἥ ∷ μ ∷ α ∷ ρ ∷ τ ∷ ε ∷ ν ∷ []) "John.9.2"
∷ word (ο ∷ ὗ ∷ τ ∷ ο ∷ ς ∷ []) "John.9.2"
∷ word (ἢ ∷ []) "John.9.2"
∷ word (ο ∷ ἱ ∷ []) "John.9.2"
∷ word (γ ∷ ο ∷ ν ∷ ε ∷ ῖ ∷ ς ∷ []) "John.9.2"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.9.2"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.9.2"
∷ word (τ ∷ υ ∷ φ ∷ ∙λ ∷ ὸ ∷ ς ∷ []) "John.9.2"
∷ word (γ ∷ ε ∷ ν ∷ ν ∷ η ∷ θ ∷ ῇ ∷ []) "John.9.2"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.9.3"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.9.3"
∷ word (Ο ∷ ὔ ∷ τ ∷ ε ∷ []) "John.9.3"
∷ word (ο ∷ ὗ ∷ τ ∷ ο ∷ ς ∷ []) "John.9.3"
∷ word (ἥ ∷ μ ∷ α ∷ ρ ∷ τ ∷ ε ∷ ν ∷ []) "John.9.3"
∷ word (ο ∷ ὔ ∷ τ ∷ ε ∷ []) "John.9.3"
∷ word (ο ∷ ἱ ∷ []) "John.9.3"
∷ word (γ ∷ ο ∷ ν ∷ ε ∷ ῖ ∷ ς ∷ []) "John.9.3"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.9.3"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ []) "John.9.3"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.9.3"
∷ word (φ ∷ α ∷ ν ∷ ε ∷ ρ ∷ ω ∷ θ ∷ ῇ ∷ []) "John.9.3"
∷ word (τ ∷ ὰ ∷ []) "John.9.3"
∷ word (ἔ ∷ ρ ∷ γ ∷ α ∷ []) "John.9.3"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.9.3"
∷ word (θ ∷ ε ∷ ο ∷ ῦ ∷ []) "John.9.3"
∷ word (ἐ ∷ ν ∷ []) "John.9.3"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.9.3"
∷ word (ἡ ∷ μ ∷ ᾶ ∷ ς ∷ []) "John.9.4"
∷ word (δ ∷ ε ∷ ῖ ∷ []) "John.9.4"
∷ word (ἐ ∷ ρ ∷ γ ∷ ά ∷ ζ ∷ ε ∷ σ ∷ θ ∷ α ∷ ι ∷ []) "John.9.4"
∷ word (τ ∷ ὰ ∷ []) "John.9.4"
∷ word (ἔ ∷ ρ ∷ γ ∷ α ∷ []) "John.9.4"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.9.4"
∷ word (π ∷ έ ∷ μ ∷ ψ ∷ α ∷ ν ∷ τ ∷ ό ∷ ς ∷ []) "John.9.4"
∷ word (μ ∷ ε ∷ []) "John.9.4"
∷ word (ἕ ∷ ω ∷ ς ∷ []) "John.9.4"
∷ word (ἡ ∷ μ ∷ έ ∷ ρ ∷ α ∷ []) "John.9.4"
∷ word (ἐ ∷ σ ∷ τ ∷ ί ∷ ν ∷ []) "John.9.4"
∷ word (ἔ ∷ ρ ∷ χ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.9.4"
∷ word (ν ∷ ὺ ∷ ξ ∷ []) "John.9.4"
∷ word (ὅ ∷ τ ∷ ε ∷ []) "John.9.4"
∷ word (ο ∷ ὐ ∷ δ ∷ ε ∷ ὶ ∷ ς ∷ []) "John.9.4"
∷ word (δ ∷ ύ ∷ ν ∷ α ∷ τ ∷ α ∷ ι ∷ []) "John.9.4"
∷ word (ἐ ∷ ρ ∷ γ ∷ ά ∷ ζ ∷ ε ∷ σ ∷ θ ∷ α ∷ ι ∷ []) "John.9.4"
∷ word (ὅ ∷ τ ∷ α ∷ ν ∷ []) "John.9.5"
∷ word (ἐ ∷ ν ∷ []) "John.9.5"
∷ word (τ ∷ ῷ ∷ []) "John.9.5"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ῳ ∷ []) "John.9.5"
∷ word (ὦ ∷ []) "John.9.5"
∷ word (φ ∷ ῶ ∷ ς ∷ []) "John.9.5"
∷ word (ε ∷ ἰ ∷ μ ∷ ι ∷ []) "John.9.5"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.9.5"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ υ ∷ []) "John.9.5"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.9.6"
∷ word (ε ∷ ἰ ∷ π ∷ ὼ ∷ ν ∷ []) "John.9.6"
∷ word (ἔ ∷ π ∷ τ ∷ υ ∷ σ ∷ ε ∷ ν ∷ []) "John.9.6"
∷ word (χ ∷ α ∷ μ ∷ α ∷ ὶ ∷ []) "John.9.6"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.9.6"
∷ word (ἐ ∷ π ∷ ο ∷ ί ∷ η ∷ σ ∷ ε ∷ ν ∷ []) "John.9.6"
∷ word (π ∷ η ∷ ∙λ ∷ ὸ ∷ ν ∷ []) "John.9.6"
∷ word (ἐ ∷ κ ∷ []) "John.9.6"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.9.6"
∷ word (π ∷ τ ∷ ύ ∷ σ ∷ μ ∷ α ∷ τ ∷ ο ∷ ς ∷ []) "John.9.6"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.9.6"
∷ word (ἐ ∷ π ∷ έ ∷ χ ∷ ρ ∷ ι ∷ σ ∷ ε ∷ ν ∷ []) "John.9.6"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.9.6"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.9.6"
∷ word (π ∷ η ∷ ∙λ ∷ ὸ ∷ ν ∷ []) "John.9.6"
∷ word (ἐ ∷ π ∷ ὶ ∷ []) "John.9.6"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.9.6"
∷ word (ὀ ∷ φ ∷ θ ∷ α ∷ ∙λ ∷ μ ∷ ο ∷ ύ ∷ ς ∷ []) "John.9.6"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.9.7"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.9.7"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.9.7"
∷ word (Ὕ ∷ π ∷ α ∷ γ ∷ ε ∷ []) "John.9.7"
∷ word (ν ∷ ί ∷ ψ ∷ α ∷ ι ∷ []) "John.9.7"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.9.7"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.9.7"
∷ word (κ ∷ ο ∷ ∙λ ∷ υ ∷ μ ∷ β ∷ ή ∷ θ ∷ ρ ∷ α ∷ ν ∷ []) "John.9.7"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.9.7"
∷ word (Σ ∷ ι ∷ ∙λ ∷ ω ∷ ά ∷ μ ∷ []) "John.9.7"
∷ word (ὃ ∷ []) "John.9.7"
∷ word (ἑ ∷ ρ ∷ μ ∷ η ∷ ν ∷ ε ∷ ύ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.9.7"
∷ word (Ἀ ∷ π ∷ ε ∷ σ ∷ τ ∷ α ∷ ∙λ ∷ μ ∷ έ ∷ ν ∷ ο ∷ ς ∷ []) "John.9.7"
∷ word (ἀ ∷ π ∷ ῆ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.9.7"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.9.7"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.9.7"
∷ word (ἐ ∷ ν ∷ ί ∷ ψ ∷ α ∷ τ ∷ ο ∷ []) "John.9.7"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.9.7"
∷ word (ἦ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.9.7"
∷ word (β ∷ ∙λ ∷ έ ∷ π ∷ ω ∷ ν ∷ []) "John.9.7"
∷ word (ο ∷ ἱ ∷ []) "John.9.8"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.9.8"
∷ word (γ ∷ ε ∷ ί ∷ τ ∷ ο ∷ ν ∷ ε ∷ ς ∷ []) "John.9.8"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.9.8"
∷ word (ο ∷ ἱ ∷ []) "John.9.8"
∷ word (θ ∷ ε ∷ ω ∷ ρ ∷ ο ∷ ῦ ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.9.8"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.9.8"
∷ word (τ ∷ ὸ ∷ []) "John.9.8"
∷ word (π ∷ ρ ∷ ό ∷ τ ∷ ε ∷ ρ ∷ ο ∷ ν ∷ []) "John.9.8"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.9.8"
∷ word (π ∷ ρ ∷ ο ∷ σ ∷ α ∷ ί ∷ τ ∷ η ∷ ς ∷ []) "John.9.8"
∷ word (ἦ ∷ ν ∷ []) "John.9.8"
∷ word (ἔ ∷ ∙λ ∷ ε ∷ γ ∷ ο ∷ ν ∷ []) "John.9.8"
∷ word (Ο ∷ ὐ ∷ χ ∷ []) "John.9.8"
∷ word (ο ∷ ὗ ∷ τ ∷ ό ∷ ς ∷ []) "John.9.8"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.9.8"
∷ word (ὁ ∷ []) "John.9.8"
∷ word (κ ∷ α ∷ θ ∷ ή ∷ μ ∷ ε ∷ ν ∷ ο ∷ ς ∷ []) "John.9.8"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.9.8"
∷ word (π ∷ ρ ∷ ο ∷ σ ∷ α ∷ ι ∷ τ ∷ ῶ ∷ ν ∷ []) "John.9.8"
∷ word (ἄ ∷ ∙λ ∷ ∙λ ∷ ο ∷ ι ∷ []) "John.9.9"
∷ word (ἔ ∷ ∙λ ∷ ε ∷ γ ∷ ο ∷ ν ∷ []) "John.9.9"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.9.9"
∷ word (Ο ∷ ὗ ∷ τ ∷ ό ∷ ς ∷ []) "John.9.9"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.9.9"
∷ word (ἄ ∷ ∙λ ∷ ∙λ ∷ ο ∷ ι ∷ []) "John.9.9"
∷ word (ἔ ∷ ∙λ ∷ ε ∷ γ ∷ ο ∷ ν ∷ []) "John.9.9"
∷ word (Ο ∷ ὐ ∷ χ ∷ ί ∷ []) "John.9.9"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.9.9"
∷ word (ὅ ∷ μ ∷ ο ∷ ι ∷ ο ∷ ς ∷ []) "John.9.9"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.9.9"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.9.9"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ο ∷ ς ∷ []) "John.9.9"
∷ word (ἔ ∷ ∙λ ∷ ε ∷ γ ∷ ε ∷ ν ∷ []) "John.9.9"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.9.9"
∷ word (Ἐ ∷ γ ∷ ώ ∷ []) "John.9.9"
∷ word (ε ∷ ἰ ∷ μ ∷ ι ∷ []) "John.9.9"
∷ word (ἔ ∷ ∙λ ∷ ε ∷ γ ∷ ο ∷ ν ∷ []) "John.9.10"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.9.10"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.9.10"
∷ word (Π ∷ ῶ ∷ ς ∷ []) "John.9.10"
∷ word (ἠ ∷ ν ∷ ε ∷ ῴ ∷ χ ∷ θ ∷ η ∷ σ ∷ ά ∷ ν ∷ []) "John.9.10"
∷ word (σ ∷ ο ∷ υ ∷ []) "John.9.10"
∷ word (ο ∷ ἱ ∷ []) "John.9.10"
∷ word (ὀ ∷ φ ∷ θ ∷ α ∷ ∙λ ∷ μ ∷ ο ∷ ί ∷ []) "John.9.10"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.9.11"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ο ∷ ς ∷ []) "John.9.11"
∷ word (Ὁ ∷ []) "John.9.11"
∷ word (ἄ ∷ ν ∷ θ ∷ ρ ∷ ω ∷ π ∷ ο ∷ ς ∷ []) "John.9.11"
∷ word (ὁ ∷ []) "John.9.11"
∷ word (∙λ ∷ ε ∷ γ ∷ ό ∷ μ ∷ ε ∷ ν ∷ ο ∷ ς ∷ []) "John.9.11"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.9.11"
∷ word (π ∷ η ∷ ∙λ ∷ ὸ ∷ ν ∷ []) "John.9.11"
∷ word (ἐ ∷ π ∷ ο ∷ ί ∷ η ∷ σ ∷ ε ∷ ν ∷ []) "John.9.11"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.9.11"
∷ word (ἐ ∷ π ∷ έ ∷ χ ∷ ρ ∷ ι ∷ σ ∷ έ ∷ ν ∷ []) "John.9.11"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.9.11"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.9.11"
∷ word (ὀ ∷ φ ∷ θ ∷ α ∷ ∙λ ∷ μ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.9.11"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.9.11"
∷ word (ε ∷ ἶ ∷ π ∷ έ ∷ ν ∷ []) "John.9.11"
∷ word (μ ∷ ο ∷ ι ∷ []) "John.9.11"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.9.11"
∷ word (Ὕ ∷ π ∷ α ∷ γ ∷ ε ∷ []) "John.9.11"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.9.11"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.9.11"
∷ word (Σ ∷ ι ∷ ∙λ ∷ ω ∷ ὰ ∷ μ ∷ []) "John.9.11"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.9.11"
∷ word (ν ∷ ί ∷ ψ ∷ α ∷ ι ∷ []) "John.9.11"
∷ word (ἀ ∷ π ∷ ε ∷ ∙λ ∷ θ ∷ ὼ ∷ ν ∷ []) "John.9.11"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.9.11"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.9.11"
∷ word (ν ∷ ι ∷ ψ ∷ ά ∷ μ ∷ ε ∷ ν ∷ ο ∷ ς ∷ []) "John.9.11"
∷ word (ἀ ∷ ν ∷ έ ∷ β ∷ ∙λ ∷ ε ∷ ψ ∷ α ∷ []) "John.9.11"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.9.12"
∷ word (ε ∷ ἶ ∷ π ∷ α ∷ ν ∷ []) "John.9.12"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.9.12"
∷ word (Π ∷ ο ∷ ῦ ∷ []) "John.9.12"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.9.12"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ο ∷ ς ∷ []) "John.9.12"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.9.12"
∷ word (Ο ∷ ὐ ∷ κ ∷ []) "John.9.12"
∷ word (ο ∷ ἶ ∷ δ ∷ α ∷ []) "John.9.12"
∷ word (Ἄ ∷ γ ∷ ο ∷ υ ∷ σ ∷ ι ∷ ν ∷ []) "John.9.13"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.9.13"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.9.13"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.9.13"
∷ word (Φ ∷ α ∷ ρ ∷ ι ∷ σ ∷ α ∷ ί ∷ ο ∷ υ ∷ ς ∷ []) "John.9.13"
∷ word (τ ∷ ό ∷ ν ∷ []) "John.9.13"
∷ word (π ∷ ο ∷ τ ∷ ε ∷ []) "John.9.13"
∷ word (τ ∷ υ ∷ φ ∷ ∙λ ∷ ό ∷ ν ∷ []) "John.9.13"
∷ word (ἦ ∷ ν ∷ []) "John.9.14"
∷ word (δ ∷ ὲ ∷ []) "John.9.14"
∷ word (σ ∷ ά ∷ β ∷ β ∷ α ∷ τ ∷ ο ∷ ν ∷ []) "John.9.14"
∷ word (ἐ ∷ ν ∷ []) "John.9.14"
∷ word (ᾗ ∷ []) "John.9.14"
∷ word (ἡ ∷ μ ∷ έ ∷ ρ ∷ ᾳ ∷ []) "John.9.14"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.9.14"
∷ word (π ∷ η ∷ ∙λ ∷ ὸ ∷ ν ∷ []) "John.9.14"
∷ word (ἐ ∷ π ∷ ο ∷ ί ∷ η ∷ σ ∷ ε ∷ ν ∷ []) "John.9.14"
∷ word (ὁ ∷ []) "John.9.14"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.9.14"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.9.14"
∷ word (ἀ ∷ ν ∷ έ ∷ ῳ ∷ ξ ∷ ε ∷ ν ∷ []) "John.9.14"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.9.14"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.9.14"
∷ word (ὀ ∷ φ ∷ θ ∷ α ∷ ∙λ ∷ μ ∷ ο ∷ ύ ∷ ς ∷ []) "John.9.14"
∷ word (π ∷ ά ∷ ∙λ ∷ ι ∷ ν ∷ []) "John.9.15"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.9.15"
∷ word (ἠ ∷ ρ ∷ ώ ∷ τ ∷ ω ∷ ν ∷ []) "John.9.15"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.9.15"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.9.15"
∷ word (ο ∷ ἱ ∷ []) "John.9.15"
∷ word (Φ ∷ α ∷ ρ ∷ ι ∷ σ ∷ α ∷ ῖ ∷ ο ∷ ι ∷ []) "John.9.15"
∷ word (π ∷ ῶ ∷ ς ∷ []) "John.9.15"
∷ word (ἀ ∷ ν ∷ έ ∷ β ∷ ∙λ ∷ ε ∷ ψ ∷ ε ∷ ν ∷ []) "John.9.15"
∷ word (ὁ ∷ []) "John.9.15"
∷ word (δ ∷ ὲ ∷ []) "John.9.15"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.9.15"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.9.15"
∷ word (Π ∷ η ∷ ∙λ ∷ ὸ ∷ ν ∷ []) "John.9.15"
∷ word (ἐ ∷ π ∷ έ ∷ θ ∷ η ∷ κ ∷ έ ∷ ν ∷ []) "John.9.15"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.9.15"
∷ word (ἐ ∷ π ∷ ὶ ∷ []) "John.9.15"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.9.15"
∷ word (ὀ ∷ φ ∷ θ ∷ α ∷ ∙λ ∷ μ ∷ ο ∷ ύ ∷ ς ∷ []) "John.9.15"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.9.15"
∷ word (ἐ ∷ ν ∷ ι ∷ ψ ∷ ά ∷ μ ∷ η ∷ ν ∷ []) "John.9.15"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.9.15"
∷ word (β ∷ ∙λ ∷ έ ∷ π ∷ ω ∷ []) "John.9.15"
∷ word (ἔ ∷ ∙λ ∷ ε ∷ γ ∷ ο ∷ ν ∷ []) "John.9.16"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.9.16"
∷ word (ἐ ∷ κ ∷ []) "John.9.16"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.9.16"
∷ word (Φ ∷ α ∷ ρ ∷ ι ∷ σ ∷ α ∷ ί ∷ ω ∷ ν ∷ []) "John.9.16"
∷ word (τ ∷ ι ∷ ν ∷ έ ∷ ς ∷ []) "John.9.16"
∷ word (Ο ∷ ὐ ∷ κ ∷ []) "John.9.16"
∷ word (ἔ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.9.16"
∷ word (ο ∷ ὗ ∷ τ ∷ ο ∷ ς ∷ []) "John.9.16"
∷ word (π ∷ α ∷ ρ ∷ ὰ ∷ []) "John.9.16"
∷ word (θ ∷ ε ∷ ο ∷ ῦ ∷ []) "John.9.16"
∷ word (ὁ ∷ []) "John.9.16"
∷ word (ἄ ∷ ν ∷ θ ∷ ρ ∷ ω ∷ π ∷ ο ∷ ς ∷ []) "John.9.16"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.9.16"
∷ word (τ ∷ ὸ ∷ []) "John.9.16"
∷ word (σ ∷ ά ∷ β ∷ β ∷ α ∷ τ ∷ ο ∷ ν ∷ []) "John.9.16"
∷ word (ο ∷ ὐ ∷ []) "John.9.16"
∷ word (τ ∷ η ∷ ρ ∷ ε ∷ ῖ ∷ []) "John.9.16"
∷ word (ἄ ∷ ∙λ ∷ ∙λ ∷ ο ∷ ι ∷ []) "John.9.16"
∷ word (ἔ ∷ ∙λ ∷ ε ∷ γ ∷ ο ∷ ν ∷ []) "John.9.16"
∷ word (Π ∷ ῶ ∷ ς ∷ []) "John.9.16"
∷ word (δ ∷ ύ ∷ ν ∷ α ∷ τ ∷ α ∷ ι ∷ []) "John.9.16"
∷ word (ἄ ∷ ν ∷ θ ∷ ρ ∷ ω ∷ π ∷ ο ∷ ς ∷ []) "John.9.16"
∷ word (ἁ ∷ μ ∷ α ∷ ρ ∷ τ ∷ ω ∷ ∙λ ∷ ὸ ∷ ς ∷ []) "John.9.16"
∷ word (τ ∷ ο ∷ ι ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.9.16"
∷ word (σ ∷ η ∷ μ ∷ ε ∷ ῖ ∷ α ∷ []) "John.9.16"
∷ word (π ∷ ο ∷ ι ∷ ε ∷ ῖ ∷ ν ∷ []) "John.9.16"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.9.16"
∷ word (σ ∷ χ ∷ ί ∷ σ ∷ μ ∷ α ∷ []) "John.9.16"
∷ word (ἦ ∷ ν ∷ []) "John.9.16"
∷ word (ἐ ∷ ν ∷ []) "John.9.16"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.9.16"
∷ word (∙λ ∷ έ ∷ γ ∷ ο ∷ υ ∷ σ ∷ ι ∷ ν ∷ []) "John.9.17"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.9.17"
∷ word (τ ∷ ῷ ∷ []) "John.9.17"
∷ word (τ ∷ υ ∷ φ ∷ ∙λ ∷ ῷ ∷ []) "John.9.17"
∷ word (π ∷ ά ∷ ∙λ ∷ ι ∷ ν ∷ []) "John.9.17"
∷ word (Τ ∷ ί ∷ []) "John.9.17"
∷ word (σ ∷ ὺ ∷ []) "John.9.17"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ ς ∷ []) "John.9.17"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.9.17"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.9.17"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.9.17"
∷ word (ἠ ∷ ν ∷ έ ∷ ῳ ∷ ξ ∷ έ ∷ ν ∷ []) "John.9.17"
∷ word (σ ∷ ο ∷ υ ∷ []) "John.9.17"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.9.17"
∷ word (ὀ ∷ φ ∷ θ ∷ α ∷ ∙λ ∷ μ ∷ ο ∷ ύ ∷ ς ∷ []) "John.9.17"
∷ word (ὁ ∷ []) "John.9.17"
∷ word (δ ∷ ὲ ∷ []) "John.9.17"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.9.17"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.9.17"
∷ word (Π ∷ ρ ∷ ο ∷ φ ∷ ή ∷ τ ∷ η ∷ ς ∷ []) "John.9.17"
∷ word (ἐ ∷ σ ∷ τ ∷ ί ∷ ν ∷ []) "John.9.17"
∷ word (Ο ∷ ὐ ∷ κ ∷ []) "John.9.18"
∷ word (ἐ ∷ π ∷ ί ∷ σ ∷ τ ∷ ε ∷ υ ∷ σ ∷ α ∷ ν ∷ []) "John.9.18"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.9.18"
∷ word (ο ∷ ἱ ∷ []) "John.9.18"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ῖ ∷ ο ∷ ι ∷ []) "John.9.18"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.9.18"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.9.18"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.9.18"
∷ word (ἦ ∷ ν ∷ []) "John.9.18"
∷ word (τ ∷ υ ∷ φ ∷ ∙λ ∷ ὸ ∷ ς ∷ []) "John.9.18"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.9.18"
∷ word (ἀ ∷ ν ∷ έ ∷ β ∷ ∙λ ∷ ε ∷ ψ ∷ ε ∷ ν ∷ []) "John.9.18"
∷ word (ἕ ∷ ω ∷ ς ∷ []) "John.9.18"
∷ word (ὅ ∷ τ ∷ ο ∷ υ ∷ []) "John.9.18"
∷ word (ἐ ∷ φ ∷ ώ ∷ ν ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.9.18"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.9.18"
∷ word (γ ∷ ο ∷ ν ∷ ε ∷ ῖ ∷ ς ∷ []) "John.9.18"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.9.18"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.9.18"
∷ word (ἀ ∷ ν ∷ α ∷ β ∷ ∙λ ∷ έ ∷ ψ ∷ α ∷ ν ∷ τ ∷ ο ∷ ς ∷ []) "John.9.18"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.9.19"
∷ word (ἠ ∷ ρ ∷ ώ ∷ τ ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.9.19"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.9.19"
∷ word (∙λ ∷ έ ∷ γ ∷ ο ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.9.19"
∷ word (Ο ∷ ὗ ∷ τ ∷ ό ∷ ς ∷ []) "John.9.19"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.9.19"
∷ word (ὁ ∷ []) "John.9.19"
∷ word (υ ∷ ἱ ∷ ὸ ∷ ς ∷ []) "John.9.19"
∷ word (ὑ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.9.19"
∷ word (ὃ ∷ ν ∷ []) "John.9.19"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.9.19"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ τ ∷ ε ∷ []) "John.9.19"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.9.19"
∷ word (τ ∷ υ ∷ φ ∷ ∙λ ∷ ὸ ∷ ς ∷ []) "John.9.19"
∷ word (ἐ ∷ γ ∷ ε ∷ ν ∷ ν ∷ ή ∷ θ ∷ η ∷ []) "John.9.19"
∷ word (π ∷ ῶ ∷ ς ∷ []) "John.9.19"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.9.19"
∷ word (β ∷ ∙λ ∷ έ ∷ π ∷ ε ∷ ι ∷ []) "John.9.19"
∷ word (ἄ ∷ ρ ∷ τ ∷ ι ∷ []) "John.9.19"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.9.20"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.9.20"
∷ word (ο ∷ ἱ ∷ []) "John.9.20"
∷ word (γ ∷ ο ∷ ν ∷ ε ∷ ῖ ∷ ς ∷ []) "John.9.20"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.9.20"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.9.20"
∷ word (ε ∷ ἶ ∷ π ∷ α ∷ ν ∷ []) "John.9.20"
∷ word (Ο ∷ ἴ ∷ δ ∷ α ∷ μ ∷ ε ∷ ν ∷ []) "John.9.20"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.9.20"
∷ word (ο ∷ ὗ ∷ τ ∷ ό ∷ ς ∷ []) "John.9.20"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.9.20"
∷ word (ὁ ∷ []) "John.9.20"
∷ word (υ ∷ ἱ ∷ ὸ ∷ ς ∷ []) "John.9.20"
∷ word (ἡ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.9.20"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.9.20"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.9.20"
∷ word (τ ∷ υ ∷ φ ∷ ∙λ ∷ ὸ ∷ ς ∷ []) "John.9.20"
∷ word (ἐ ∷ γ ∷ ε ∷ ν ∷ ν ∷ ή ∷ θ ∷ η ∷ []) "John.9.20"
∷ word (π ∷ ῶ ∷ ς ∷ []) "John.9.21"
∷ word (δ ∷ ὲ ∷ []) "John.9.21"
∷ word (ν ∷ ῦ ∷ ν ∷ []) "John.9.21"
∷ word (β ∷ ∙λ ∷ έ ∷ π ∷ ε ∷ ι ∷ []) "John.9.21"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.9.21"
∷ word (ο ∷ ἴ ∷ δ ∷ α ∷ μ ∷ ε ∷ ν ∷ []) "John.9.21"
∷ word (ἢ ∷ []) "John.9.21"
∷ word (τ ∷ ί ∷ ς ∷ []) "John.9.21"
∷ word (ἤ ∷ ν ∷ ο ∷ ι ∷ ξ ∷ ε ∷ ν ∷ []) "John.9.21"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.9.21"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.9.21"
∷ word (ὀ ∷ φ ∷ θ ∷ α ∷ ∙λ ∷ μ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.9.21"
∷ word (ἡ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.9.21"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.9.21"
∷ word (ο ∷ ἴ ∷ δ ∷ α ∷ μ ∷ ε ∷ ν ∷ []) "John.9.21"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.9.21"
∷ word (ἐ ∷ ρ ∷ ω ∷ τ ∷ ή ∷ σ ∷ α ∷ τ ∷ ε ∷ []) "John.9.21"
∷ word (ἡ ∷ ∙λ ∷ ι ∷ κ ∷ ί ∷ α ∷ ν ∷ []) "John.9.21"
∷ word (ἔ ∷ χ ∷ ε ∷ ι ∷ []) "John.9.21"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ς ∷ []) "John.9.21"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.9.21"
∷ word (ἑ ∷ α ∷ υ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.9.21"
∷ word (∙λ ∷ α ∷ ∙λ ∷ ή ∷ σ ∷ ε ∷ ι ∷ []) "John.9.21"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.9.22"
∷ word (ε ∷ ἶ ∷ π ∷ α ∷ ν ∷ []) "John.9.22"
∷ word (ο ∷ ἱ ∷ []) "John.9.22"
∷ word (γ ∷ ο ∷ ν ∷ ε ∷ ῖ ∷ ς ∷ []) "John.9.22"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.9.22"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.9.22"
∷ word (ἐ ∷ φ ∷ ο ∷ β ∷ ο ∷ ῦ ∷ ν ∷ τ ∷ ο ∷ []) "John.9.22"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.9.22"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ί ∷ ο ∷ υ ∷ ς ∷ []) "John.9.22"
∷ word (ἤ ∷ δ ∷ η ∷ []) "John.9.22"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.9.22"
∷ word (σ ∷ υ ∷ ν ∷ ε ∷ τ ∷ έ ∷ θ ∷ ε ∷ ι ∷ ν ∷ τ ∷ ο ∷ []) "John.9.22"
∷ word (ο ∷ ἱ ∷ []) "John.9.22"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ῖ ∷ ο ∷ ι ∷ []) "John.9.22"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.9.22"
∷ word (ἐ ∷ ά ∷ ν ∷ []) "John.9.22"
∷ word (τ ∷ ι ∷ ς ∷ []) "John.9.22"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.9.22"
∷ word (ὁ ∷ μ ∷ ο ∷ ∙λ ∷ ο ∷ γ ∷ ή ∷ σ ∷ ῃ ∷ []) "John.9.22"
∷ word (χ ∷ ρ ∷ ι ∷ σ ∷ τ ∷ ό ∷ ν ∷ []) "John.9.22"
∷ word (ἀ ∷ π ∷ ο ∷ σ ∷ υ ∷ ν ∷ ά ∷ γ ∷ ω ∷ γ ∷ ο ∷ ς ∷ []) "John.9.22"
∷ word (γ ∷ έ ∷ ν ∷ η ∷ τ ∷ α ∷ ι ∷ []) "John.9.22"
∷ word (δ ∷ ι ∷ ὰ ∷ []) "John.9.23"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.9.23"
∷ word (ο ∷ ἱ ∷ []) "John.9.23"
∷ word (γ ∷ ο ∷ ν ∷ ε ∷ ῖ ∷ ς ∷ []) "John.9.23"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.9.23"
∷ word (ε ∷ ἶ ∷ π ∷ α ∷ ν ∷ []) "John.9.23"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.9.23"
∷ word (Ἡ ∷ ∙λ ∷ ι ∷ κ ∷ ί ∷ α ∷ ν ∷ []) "John.9.23"
∷ word (ἔ ∷ χ ∷ ε ∷ ι ∷ []) "John.9.23"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.9.23"
∷ word (ἐ ∷ π ∷ ε ∷ ρ ∷ ω ∷ τ ∷ ή ∷ σ ∷ α ∷ τ ∷ ε ∷ []) "John.9.23"
∷ word (Ἐ ∷ φ ∷ ώ ∷ ν ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.9.24"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.9.24"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.9.24"
∷ word (ἄ ∷ ν ∷ θ ∷ ρ ∷ ω ∷ π ∷ ο ∷ ν ∷ []) "John.9.24"
∷ word (ἐ ∷ κ ∷ []) "John.9.24"
∷ word (δ ∷ ε ∷ υ ∷ τ ∷ έ ∷ ρ ∷ ο ∷ υ ∷ []) "John.9.24"
∷ word (ὃ ∷ ς ∷ []) "John.9.24"
∷ word (ἦ ∷ ν ∷ []) "John.9.24"
∷ word (τ ∷ υ ∷ φ ∷ ∙λ ∷ ὸ ∷ ς ∷ []) "John.9.24"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.9.24"
∷ word (ε ∷ ἶ ∷ π ∷ α ∷ ν ∷ []) "John.9.24"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.9.24"
∷ word (Δ ∷ ὸ ∷ ς ∷ []) "John.9.24"
∷ word (δ ∷ ό ∷ ξ ∷ α ∷ ν ∷ []) "John.9.24"
∷ word (τ ∷ ῷ ∷ []) "John.9.24"
∷ word (θ ∷ ε ∷ ῷ ∷ []) "John.9.24"
∷ word (ἡ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.9.24"
∷ word (ο ∷ ἴ ∷ δ ∷ α ∷ μ ∷ ε ∷ ν ∷ []) "John.9.24"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.9.24"
∷ word (ο ∷ ὗ ∷ τ ∷ ο ∷ ς ∷ []) "John.9.24"
∷ word (ὁ ∷ []) "John.9.24"
∷ word (ἄ ∷ ν ∷ θ ∷ ρ ∷ ω ∷ π ∷ ο ∷ ς ∷ []) "John.9.24"
∷ word (ἁ ∷ μ ∷ α ∷ ρ ∷ τ ∷ ω ∷ ∙λ ∷ ό ∷ ς ∷ []) "John.9.24"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.9.24"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.9.25"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.9.25"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ο ∷ ς ∷ []) "John.9.25"
∷ word (Ε ∷ ἰ ∷ []) "John.9.25"
∷ word (ἁ ∷ μ ∷ α ∷ ρ ∷ τ ∷ ω ∷ ∙λ ∷ ό ∷ ς ∷ []) "John.9.25"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.9.25"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.9.25"
∷ word (ο ∷ ἶ ∷ δ ∷ α ∷ []) "John.9.25"
∷ word (ἓ ∷ ν ∷ []) "John.9.25"
∷ word (ο ∷ ἶ ∷ δ ∷ α ∷ []) "John.9.25"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.9.25"
∷ word (τ ∷ υ ∷ φ ∷ ∙λ ∷ ὸ ∷ ς ∷ []) "John.9.25"
∷ word (ὢ ∷ ν ∷ []) "John.9.25"
∷ word (ἄ ∷ ρ ∷ τ ∷ ι ∷ []) "John.9.25"
∷ word (β ∷ ∙λ ∷ έ ∷ π ∷ ω ∷ []) "John.9.25"
∷ word (ε ∷ ἶ ∷ π ∷ ο ∷ ν ∷ []) "John.9.26"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.9.26"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.9.26"
∷ word (Τ ∷ ί ∷ []) "John.9.26"
∷ word (ἐ ∷ π ∷ ο ∷ ί ∷ η ∷ σ ∷ έ ∷ ν ∷ []) "John.9.26"
∷ word (σ ∷ ο ∷ ι ∷ []) "John.9.26"
∷ word (π ∷ ῶ ∷ ς ∷ []) "John.9.26"
∷ word (ἤ ∷ ν ∷ ο ∷ ι ∷ ξ ∷ έ ∷ ν ∷ []) "John.9.26"
∷ word (σ ∷ ο ∷ υ ∷ []) "John.9.26"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.9.26"
∷ word (ὀ ∷ φ ∷ θ ∷ α ∷ ∙λ ∷ μ ∷ ο ∷ ύ ∷ ς ∷ []) "John.9.26"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.9.27"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.9.27"
∷ word (Ε ∷ ἶ ∷ π ∷ ο ∷ ν ∷ []) "John.9.27"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.9.27"
∷ word (ἤ ∷ δ ∷ η ∷ []) "John.9.27"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.9.27"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.9.27"
∷ word (ἠ ∷ κ ∷ ο ∷ ύ ∷ σ ∷ α ∷ τ ∷ ε ∷ []) "John.9.27"
∷ word (τ ∷ ί ∷ []) "John.9.27"
∷ word (π ∷ ά ∷ ∙λ ∷ ι ∷ ν ∷ []) "John.9.27"
∷ word (θ ∷ έ ∷ ∙λ ∷ ε ∷ τ ∷ ε ∷ []) "John.9.27"
∷ word (ἀ ∷ κ ∷ ο ∷ ύ ∷ ε ∷ ι ∷ ν ∷ []) "John.9.27"
∷ word (μ ∷ ὴ ∷ []) "John.9.27"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.9.27"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.9.27"
∷ word (θ ∷ έ ∷ ∙λ ∷ ε ∷ τ ∷ ε ∷ []) "John.9.27"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.9.27"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ α ∷ ὶ ∷ []) "John.9.27"
∷ word (γ ∷ ε ∷ ν ∷ έ ∷ σ ∷ θ ∷ α ∷ ι ∷ []) "John.9.27"
∷ word (ἐ ∷ ∙λ ∷ ο ∷ ι ∷ δ ∷ ό ∷ ρ ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.9.28"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.9.28"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.9.28"
∷ word (ε ∷ ἶ ∷ π ∷ ο ∷ ν ∷ []) "John.9.28"
∷ word (Σ ∷ ὺ ∷ []) "John.9.28"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ ὴ ∷ ς ∷ []) "John.9.28"
∷ word (ε ∷ ἶ ∷ []) "John.9.28"
∷ word (ἐ ∷ κ ∷ ε ∷ ί ∷ ν ∷ ο ∷ υ ∷ []) "John.9.28"
∷ word (ἡ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.9.28"
∷ word (δ ∷ ὲ ∷ []) "John.9.28"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.9.28"
∷ word (Μ ∷ ω ∷ ϋ ∷ σ ∷ έ ∷ ω ∷ ς ∷ []) "John.9.28"
∷ word (ἐ ∷ σ ∷ μ ∷ ὲ ∷ ν ∷ []) "John.9.28"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ α ∷ ί ∷ []) "John.9.28"
∷ word (ἡ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.9.29"
∷ word (ο ∷ ἴ ∷ δ ∷ α ∷ μ ∷ ε ∷ ν ∷ []) "John.9.29"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.9.29"
∷ word (Μ ∷ ω ∷ ϋ ∷ σ ∷ ε ∷ ῖ ∷ []) "John.9.29"
∷ word (∙λ ∷ ε ∷ ∙λ ∷ ά ∷ ∙λ ∷ η ∷ κ ∷ ε ∷ ν ∷ []) "John.9.29"
∷ word (ὁ ∷ []) "John.9.29"
∷ word (θ ∷ ε ∷ ό ∷ ς ∷ []) "John.9.29"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ ν ∷ []) "John.9.29"
∷ word (δ ∷ ὲ ∷ []) "John.9.29"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.9.29"
∷ word (ο ∷ ἴ ∷ δ ∷ α ∷ μ ∷ ε ∷ ν ∷ []) "John.9.29"
∷ word (π ∷ ό ∷ θ ∷ ε ∷ ν ∷ []) "John.9.29"
∷ word (ἐ ∷ σ ∷ τ ∷ ί ∷ ν ∷ []) "John.9.29"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.9.30"
∷ word (ὁ ∷ []) "John.9.30"
∷ word (ἄ ∷ ν ∷ θ ∷ ρ ∷ ω ∷ π ∷ ο ∷ ς ∷ []) "John.9.30"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.9.30"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.9.30"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.9.30"
∷ word (Ἐ ∷ ν ∷ []) "John.9.30"
∷ word (τ ∷ ο ∷ ύ ∷ τ ∷ ῳ ∷ []) "John.9.30"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.9.30"
∷ word (τ ∷ ὸ ∷ []) "John.9.30"
∷ word (θ ∷ α ∷ υ ∷ μ ∷ α ∷ σ ∷ τ ∷ ό ∷ ν ∷ []) "John.9.30"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.9.30"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.9.30"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.9.30"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.9.30"
∷ word (ο ∷ ἴ ∷ δ ∷ α ∷ τ ∷ ε ∷ []) "John.9.30"
∷ word (π ∷ ό ∷ θ ∷ ε ∷ ν ∷ []) "John.9.30"
∷ word (ἐ ∷ σ ∷ τ ∷ ί ∷ ν ∷ []) "John.9.30"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.9.30"
∷ word (ἤ ∷ ν ∷ ο ∷ ι ∷ ξ ∷ έ ∷ ν ∷ []) "John.9.30"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.9.30"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.9.30"
∷ word (ὀ ∷ φ ∷ θ ∷ α ∷ ∙λ ∷ μ ∷ ο ∷ ύ ∷ ς ∷ []) "John.9.30"
∷ word (ο ∷ ἴ ∷ δ ∷ α ∷ μ ∷ ε ∷ ν ∷ []) "John.9.31"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.9.31"
∷ word (ἁ ∷ μ ∷ α ∷ ρ ∷ τ ∷ ω ∷ ∙λ ∷ ῶ ∷ ν ∷ []) "John.9.31"
∷ word (ὁ ∷ []) "John.9.31"
∷ word (θ ∷ ε ∷ ὸ ∷ ς ∷ []) "John.9.31"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.9.31"
∷ word (ἀ ∷ κ ∷ ο ∷ ύ ∷ ε ∷ ι ∷ []) "John.9.31"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ []) "John.9.31"
∷ word (ἐ ∷ ά ∷ ν ∷ []) "John.9.31"
∷ word (τ ∷ ι ∷ ς ∷ []) "John.9.31"
∷ word (θ ∷ ε ∷ ο ∷ σ ∷ ε ∷ β ∷ ὴ ∷ ς ∷ []) "John.9.31"
∷ word (ᾖ ∷ []) "John.9.31"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.9.31"
∷ word (τ ∷ ὸ ∷ []) "John.9.31"
∷ word (θ ∷ έ ∷ ∙λ ∷ η ∷ μ ∷ α ∷ []) "John.9.31"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.9.31"
∷ word (π ∷ ο ∷ ι ∷ ῇ ∷ []) "John.9.31"
∷ word (τ ∷ ο ∷ ύ ∷ τ ∷ ο ∷ υ ∷ []) "John.9.31"
∷ word (ἀ ∷ κ ∷ ο ∷ ύ ∷ ε ∷ ι ∷ []) "John.9.31"
∷ word (ἐ ∷ κ ∷ []) "John.9.32"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.9.32"
∷ word (α ∷ ἰ ∷ ῶ ∷ ν ∷ ο ∷ ς ∷ []) "John.9.32"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.9.32"
∷ word (ἠ ∷ κ ∷ ο ∷ ύ ∷ σ ∷ θ ∷ η ∷ []) "John.9.32"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.9.32"
∷ word (ἠ ∷ ν ∷ έ ∷ ῳ ∷ ξ ∷ έ ∷ ν ∷ []) "John.9.32"
∷ word (τ ∷ ι ∷ ς ∷ []) "John.9.32"
∷ word (ὀ ∷ φ ∷ θ ∷ α ∷ ∙λ ∷ μ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.9.32"
∷ word (τ ∷ υ ∷ φ ∷ ∙λ ∷ ο ∷ ῦ ∷ []) "John.9.32"
∷ word (γ ∷ ε ∷ γ ∷ ε ∷ ν ∷ ν ∷ η ∷ μ ∷ έ ∷ ν ∷ ο ∷ υ ∷ []) "John.9.32"
∷ word (ε ∷ ἰ ∷ []) "John.9.33"
∷ word (μ ∷ ὴ ∷ []) "John.9.33"
∷ word (ἦ ∷ ν ∷ []) "John.9.33"
∷ word (ο ∷ ὗ ∷ τ ∷ ο ∷ ς ∷ []) "John.9.33"
∷ word (π ∷ α ∷ ρ ∷ ὰ ∷ []) "John.9.33"
∷ word (θ ∷ ε ∷ ο ∷ ῦ ∷ []) "John.9.33"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.9.33"
∷ word (ἠ ∷ δ ∷ ύ ∷ ν ∷ α ∷ τ ∷ ο ∷ []) "John.9.33"
∷ word (π ∷ ο ∷ ι ∷ ε ∷ ῖ ∷ ν ∷ []) "John.9.33"
∷ word (ο ∷ ὐ ∷ δ ∷ έ ∷ ν ∷ []) "John.9.33"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.9.34"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.9.34"
∷ word (ε ∷ ἶ ∷ π ∷ α ∷ ν ∷ []) "John.9.34"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.9.34"
∷ word (Ἐ ∷ ν ∷ []) "John.9.34"
∷ word (ἁ ∷ μ ∷ α ∷ ρ ∷ τ ∷ ί ∷ α ∷ ι ∷ ς ∷ []) "John.9.34"
∷ word (σ ∷ ὺ ∷ []) "John.9.34"
∷ word (ἐ ∷ γ ∷ ε ∷ ν ∷ ν ∷ ή ∷ θ ∷ η ∷ ς ∷ []) "John.9.34"
∷ word (ὅ ∷ ∙λ ∷ ο ∷ ς ∷ []) "John.9.34"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.9.34"
∷ word (σ ∷ ὺ ∷ []) "John.9.34"
∷ word (δ ∷ ι ∷ δ ∷ ά ∷ σ ∷ κ ∷ ε ∷ ι ∷ ς ∷ []) "John.9.34"
∷ word (ἡ ∷ μ ∷ ᾶ ∷ ς ∷ []) "John.9.34"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.9.34"
∷ word (ἐ ∷ ξ ∷ έ ∷ β ∷ α ∷ ∙λ ∷ ο ∷ ν ∷ []) "John.9.34"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.9.34"
∷ word (ἔ ∷ ξ ∷ ω ∷ []) "John.9.34"
∷ word (Ἤ ∷ κ ∷ ο ∷ υ ∷ σ ∷ ε ∷ ν ∷ []) "John.9.35"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.9.35"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.9.35"
∷ word (ἐ ∷ ξ ∷ έ ∷ β ∷ α ∷ ∙λ ∷ ο ∷ ν ∷ []) "John.9.35"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.9.35"
∷ word (ἔ ∷ ξ ∷ ω ∷ []) "John.9.35"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.9.35"
∷ word (ε ∷ ὑ ∷ ρ ∷ ὼ ∷ ν ∷ []) "John.9.35"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.9.35"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.9.35"
∷ word (Σ ∷ ὺ ∷ []) "John.9.35"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ ε ∷ ι ∷ ς ∷ []) "John.9.35"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.9.35"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.9.35"
∷ word (υ ∷ ἱ ∷ ὸ ∷ ν ∷ []) "John.9.35"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.9.35"
∷ word (ἀ ∷ ν ∷ θ ∷ ρ ∷ ώ ∷ π ∷ ο ∷ υ ∷ []) "John.9.35"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.9.36"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ο ∷ ς ∷ []) "John.9.36"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.9.36"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.9.36"
∷ word (Κ ∷ α ∷ ὶ ∷ []) "John.9.36"
∷ word (τ ∷ ί ∷ ς ∷ []) "John.9.36"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.9.36"
∷ word (κ ∷ ύ ∷ ρ ∷ ι ∷ ε ∷ []) "John.9.36"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.9.36"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ σ ∷ ω ∷ []) "John.9.36"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.9.36"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.9.36"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.9.37"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.9.37"
∷ word (ὁ ∷ []) "John.9.37"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.9.37"
∷ word (Κ ∷ α ∷ ὶ ∷ []) "John.9.37"
∷ word (ἑ ∷ ώ ∷ ρ ∷ α ∷ κ ∷ α ∷ ς ∷ []) "John.9.37"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.9.37"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.9.37"
∷ word (ὁ ∷ []) "John.9.37"
∷ word (∙λ ∷ α ∷ ∙λ ∷ ῶ ∷ ν ∷ []) "John.9.37"
∷ word (μ ∷ ε ∷ τ ∷ ὰ ∷ []) "John.9.37"
∷ word (σ ∷ ο ∷ ῦ ∷ []) "John.9.37"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ό ∷ ς ∷ []) "John.9.37"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.9.37"
∷ word (ὁ ∷ []) "John.9.38"
∷ word (δ ∷ ὲ ∷ []) "John.9.38"
∷ word (ἔ ∷ φ ∷ η ∷ []) "John.9.38"
∷ word (Π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ ω ∷ []) "John.9.38"
∷ word (κ ∷ ύ ∷ ρ ∷ ι ∷ ε ∷ []) "John.9.38"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.9.38"
∷ word (π ∷ ρ ∷ ο ∷ σ ∷ ε ∷ κ ∷ ύ ∷ ν ∷ η ∷ σ ∷ ε ∷ ν ∷ []) "John.9.38"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.9.38"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.9.39"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.9.39"
∷ word (ὁ ∷ []) "John.9.39"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.9.39"
∷ word (Ε ∷ ἰ ∷ ς ∷ []) "John.9.39"
∷ word (κ ∷ ρ ∷ ί ∷ μ ∷ α ∷ []) "John.9.39"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.9.39"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.9.39"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.9.39"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ ν ∷ []) "John.9.39"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ ν ∷ []) "John.9.39"
∷ word (ἦ ∷ ∙λ ∷ θ ∷ ο ∷ ν ∷ []) "John.9.39"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.9.39"
∷ word (ο ∷ ἱ ∷ []) "John.9.39"
∷ word (μ ∷ ὴ ∷ []) "John.9.39"
∷ word (β ∷ ∙λ ∷ έ ∷ π ∷ ο ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.9.39"
∷ word (β ∷ ∙λ ∷ έ ∷ π ∷ ω ∷ σ ∷ ι ∷ ν ∷ []) "John.9.39"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.9.39"
∷ word (ο ∷ ἱ ∷ []) "John.9.39"
∷ word (β ∷ ∙λ ∷ έ ∷ π ∷ ο ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.9.39"
∷ word (τ ∷ υ ∷ φ ∷ ∙λ ∷ ο ∷ ὶ ∷ []) "John.9.39"
∷ word (γ ∷ έ ∷ ν ∷ ω ∷ ν ∷ τ ∷ α ∷ ι ∷ []) "John.9.39"
∷ word (ἤ ∷ κ ∷ ο ∷ υ ∷ σ ∷ α ∷ ν ∷ []) "John.9.40"
∷ word (ἐ ∷ κ ∷ []) "John.9.40"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.9.40"
∷ word (Φ ∷ α ∷ ρ ∷ ι ∷ σ ∷ α ∷ ί ∷ ω ∷ ν ∷ []) "John.9.40"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.9.40"
∷ word (ο ∷ ἱ ∷ []) "John.9.40"
∷ word (μ ∷ ε ∷ τ ∷ []) "John.9.40"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.9.40"
∷ word (ὄ ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.9.40"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.9.40"
∷ word (ε ∷ ἶ ∷ π ∷ ο ∷ ν ∷ []) "John.9.40"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.9.40"
∷ word (Μ ∷ ὴ ∷ []) "John.9.40"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.9.40"
∷ word (ἡ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.9.40"
∷ word (τ ∷ υ ∷ φ ∷ ∙λ ∷ ο ∷ ί ∷ []) "John.9.40"
∷ word (ἐ ∷ σ ∷ μ ∷ ε ∷ ν ∷ []) "John.9.40"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.9.41"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.9.41"
∷ word (ὁ ∷ []) "John.9.41"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.9.41"
∷ word (Ε ∷ ἰ ∷ []) "John.9.41"
∷ word (τ ∷ υ ∷ φ ∷ ∙λ ∷ ο ∷ ὶ ∷ []) "John.9.41"
∷ word (ἦ ∷ τ ∷ ε ∷ []) "John.9.41"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.9.41"
∷ word (ἂ ∷ ν ∷ []) "John.9.41"
∷ word (ε ∷ ἴ ∷ χ ∷ ε ∷ τ ∷ ε ∷ []) "John.9.41"
∷ word (ἁ ∷ μ ∷ α ∷ ρ ∷ τ ∷ ί ∷ α ∷ ν ∷ []) "John.9.41"
∷ word (ν ∷ ῦ ∷ ν ∷ []) "John.9.41"
∷ word (δ ∷ ὲ ∷ []) "John.9.41"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ τ ∷ ε ∷ []) "John.9.41"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.9.41"
∷ word (Β ∷ ∙λ ∷ έ ∷ π ∷ ο ∷ μ ∷ ε ∷ ν ∷ []) "John.9.41"
∷ word (ἡ ∷ []) "John.9.41"
∷ word (ἁ ∷ μ ∷ α ∷ ρ ∷ τ ∷ ί ∷ α ∷ []) "John.9.41"
∷ word (ὑ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.9.41"
∷ word (μ ∷ έ ∷ ν ∷ ε ∷ ι ∷ []) "John.9.41"
∷ word (Ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.10.1"
∷ word (ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.10.1"
∷ word (∙λ ∷ έ ∷ γ ∷ ω ∷ []) "John.10.1"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.10.1"
∷ word (ὁ ∷ []) "John.10.1"
∷ word (μ ∷ ὴ ∷ []) "John.10.1"
∷ word (ε ∷ ἰ ∷ σ ∷ ε ∷ ρ ∷ χ ∷ ό ∷ μ ∷ ε ∷ ν ∷ ο ∷ ς ∷ []) "John.10.1"
∷ word (δ ∷ ι ∷ ὰ ∷ []) "John.10.1"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.10.1"
∷ word (θ ∷ ύ ∷ ρ ∷ α ∷ ς ∷ []) "John.10.1"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.10.1"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.10.1"
∷ word (α ∷ ὐ ∷ ∙λ ∷ ὴ ∷ ν ∷ []) "John.10.1"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.10.1"
∷ word (π ∷ ρ ∷ ο ∷ β ∷ ά ∷ τ ∷ ω ∷ ν ∷ []) "John.10.1"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.10.1"
∷ word (ἀ ∷ ν ∷ α ∷ β ∷ α ∷ ί ∷ ν ∷ ω ∷ ν ∷ []) "John.10.1"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ α ∷ χ ∷ ό ∷ θ ∷ ε ∷ ν ∷ []) "John.10.1"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ο ∷ ς ∷ []) "John.10.1"
∷ word (κ ∷ ∙λ ∷ έ ∷ π ∷ τ ∷ η ∷ ς ∷ []) "John.10.1"
∷ word (ἐ ∷ σ ∷ τ ∷ ὶ ∷ ν ∷ []) "John.10.1"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.10.1"
∷ word (∙λ ∷ ῃ ∷ σ ∷ τ ∷ ή ∷ ς ∷ []) "John.10.1"
∷ word (ὁ ∷ []) "John.10.2"
∷ word (δ ∷ ὲ ∷ []) "John.10.2"
∷ word (ε ∷ ἰ ∷ σ ∷ ε ∷ ρ ∷ χ ∷ ό ∷ μ ∷ ε ∷ ν ∷ ο ∷ ς ∷ []) "John.10.2"
∷ word (δ ∷ ι ∷ ὰ ∷ []) "John.10.2"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.10.2"
∷ word (θ ∷ ύ ∷ ρ ∷ α ∷ ς ∷ []) "John.10.2"
∷ word (π ∷ ο ∷ ι ∷ μ ∷ ή ∷ ν ∷ []) "John.10.2"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.10.2"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.10.2"
∷ word (π ∷ ρ ∷ ο ∷ β ∷ ά ∷ τ ∷ ω ∷ ν ∷ []) "John.10.2"
∷ word (τ ∷ ο ∷ ύ ∷ τ ∷ ῳ ∷ []) "John.10.3"
∷ word (ὁ ∷ []) "John.10.3"
∷ word (θ ∷ υ ∷ ρ ∷ ω ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.10.3"
∷ word (ἀ ∷ ν ∷ ο ∷ ί ∷ γ ∷ ε ∷ ι ∷ []) "John.10.3"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.10.3"
∷ word (τ ∷ ὰ ∷ []) "John.10.3"
∷ word (π ∷ ρ ∷ ό ∷ β ∷ α ∷ τ ∷ α ∷ []) "John.10.3"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.10.3"
∷ word (φ ∷ ω ∷ ν ∷ ῆ ∷ ς ∷ []) "John.10.3"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.10.3"
∷ word (ἀ ∷ κ ∷ ο ∷ ύ ∷ ε ∷ ι ∷ []) "John.10.3"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.10.3"
∷ word (τ ∷ ὰ ∷ []) "John.10.3"
∷ word (ἴ ∷ δ ∷ ι ∷ α ∷ []) "John.10.3"
∷ word (π ∷ ρ ∷ ό ∷ β ∷ α ∷ τ ∷ α ∷ []) "John.10.3"
∷ word (φ ∷ ω ∷ ν ∷ ε ∷ ῖ ∷ []) "John.10.3"
∷ word (κ ∷ α ∷ τ ∷ []) "John.10.3"
∷ word (ὄ ∷ ν ∷ ο ∷ μ ∷ α ∷ []) "John.10.3"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.10.3"
∷ word (ἐ ∷ ξ ∷ ά ∷ γ ∷ ε ∷ ι ∷ []) "John.10.3"
∷ word (α ∷ ὐ ∷ τ ∷ ά ∷ []) "John.10.3"
∷ word (ὅ ∷ τ ∷ α ∷ ν ∷ []) "John.10.4"
∷ word (τ ∷ ὰ ∷ []) "John.10.4"
∷ word (ἴ ∷ δ ∷ ι ∷ α ∷ []) "John.10.4"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ α ∷ []) "John.10.4"
∷ word (ἐ ∷ κ ∷ β ∷ ά ∷ ∙λ ∷ ῃ ∷ []) "John.10.4"
∷ word (ἔ ∷ μ ∷ π ∷ ρ ∷ ο ∷ σ ∷ θ ∷ ε ∷ ν ∷ []) "John.10.4"
∷ word (α ∷ ὐ ∷ τ ∷ ῶ ∷ ν ∷ []) "John.10.4"
∷ word (π ∷ ο ∷ ρ ∷ ε ∷ ύ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.10.4"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.10.4"
∷ word (τ ∷ ὰ ∷ []) "John.10.4"
∷ word (π ∷ ρ ∷ ό ∷ β ∷ α ∷ τ ∷ α ∷ []) "John.10.4"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.10.4"
∷ word (ἀ ∷ κ ∷ ο ∷ ∙λ ∷ ο ∷ υ ∷ θ ∷ ε ∷ ῖ ∷ []) "John.10.4"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.10.4"
∷ word (ο ∷ ἴ ∷ δ ∷ α ∷ σ ∷ ι ∷ ν ∷ []) "John.10.4"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.10.4"
∷ word (φ ∷ ω ∷ ν ∷ ὴ ∷ ν ∷ []) "John.10.4"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.10.4"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ο ∷ τ ∷ ρ ∷ ί ∷ ῳ ∷ []) "John.10.5"
∷ word (δ ∷ ὲ ∷ []) "John.10.5"
∷ word (ο ∷ ὐ ∷ []) "John.10.5"
∷ word (μ ∷ ὴ ∷ []) "John.10.5"
∷ word (ἀ ∷ κ ∷ ο ∷ ∙λ ∷ ο ∷ υ ∷ θ ∷ ή ∷ σ ∷ ο ∷ υ ∷ σ ∷ ι ∷ ν ∷ []) "John.10.5"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.10.5"
∷ word (φ ∷ ε ∷ ύ ∷ ξ ∷ ο ∷ ν ∷ τ ∷ α ∷ ι ∷ []) "John.10.5"
∷ word (ἀ ∷ π ∷ []) "John.10.5"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.10.5"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.10.5"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.10.5"
∷ word (ο ∷ ἴ ∷ δ ∷ α ∷ σ ∷ ι ∷ []) "John.10.5"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.10.5"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ο ∷ τ ∷ ρ ∷ ί ∷ ω ∷ ν ∷ []) "John.10.5"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.10.5"
∷ word (φ ∷ ω ∷ ν ∷ ή ∷ ν ∷ []) "John.10.5"
∷ word (τ ∷ α ∷ ύ ∷ τ ∷ η ∷ ν ∷ []) "John.10.6"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.10.6"
∷ word (π ∷ α ∷ ρ ∷ ο ∷ ι ∷ μ ∷ ί ∷ α ∷ ν ∷ []) "John.10.6"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.10.6"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.10.6"
∷ word (ὁ ∷ []) "John.10.6"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.10.6"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ο ∷ ι ∷ []) "John.10.6"
∷ word (δ ∷ ὲ ∷ []) "John.10.6"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.10.6"
∷ word (ἔ ∷ γ ∷ ν ∷ ω ∷ σ ∷ α ∷ ν ∷ []) "John.10.6"
∷ word (τ ∷ ί ∷ ν ∷ α ∷ []) "John.10.6"
∷ word (ἦ ∷ ν ∷ []) "John.10.6"
∷ word (ἃ ∷ []) "John.10.6"
∷ word (ἐ ∷ ∙λ ∷ ά ∷ ∙λ ∷ ε ∷ ι ∷ []) "John.10.6"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.10.6"
∷ word (Ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.10.7"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.10.7"
∷ word (π ∷ ά ∷ ∙λ ∷ ι ∷ ν ∷ []) "John.10.7"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.10.7"
∷ word (ὁ ∷ []) "John.10.7"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.10.7"
∷ word (Ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.10.7"
∷ word (ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.10.7"
∷ word (∙λ ∷ έ ∷ γ ∷ ω ∷ []) "John.10.7"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.10.7"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.10.7"
∷ word (ἐ ∷ γ ∷ ώ ∷ []) "John.10.7"
∷ word (ε ∷ ἰ ∷ μ ∷ ι ∷ []) "John.10.7"
∷ word (ἡ ∷ []) "John.10.7"
∷ word (θ ∷ ύ ∷ ρ ∷ α ∷ []) "John.10.7"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.10.7"
∷ word (π ∷ ρ ∷ ο ∷ β ∷ ά ∷ τ ∷ ω ∷ ν ∷ []) "John.10.7"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.10.8"
∷ word (ὅ ∷ σ ∷ ο ∷ ι ∷ []) "John.10.8"
∷ word (ἦ ∷ ∙λ ∷ θ ∷ ο ∷ ν ∷ []) "John.10.8"
∷ word (π ∷ ρ ∷ ὸ ∷ []) "John.10.8"
∷ word (ἐ ∷ μ ∷ ο ∷ ῦ ∷ []) "John.10.8"
∷ word (κ ∷ ∙λ ∷ έ ∷ π ∷ τ ∷ α ∷ ι ∷ []) "John.10.8"
∷ word (ε ∷ ἰ ∷ σ ∷ ὶ ∷ ν ∷ []) "John.10.8"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.10.8"
∷ word (∙λ ∷ ῃ ∷ σ ∷ τ ∷ α ∷ ί ∷ []) "John.10.8"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ []) "John.10.8"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.10.8"
∷ word (ἤ ∷ κ ∷ ο ∷ υ ∷ σ ∷ α ∷ ν ∷ []) "John.10.8"
∷ word (α ∷ ὐ ∷ τ ∷ ῶ ∷ ν ∷ []) "John.10.8"
∷ word (τ ∷ ὰ ∷ []) "John.10.8"
∷ word (π ∷ ρ ∷ ό ∷ β ∷ α ∷ τ ∷ α ∷ []) "John.10.8"
∷ word (ἐ ∷ γ ∷ ώ ∷ []) "John.10.9"
∷ word (ε ∷ ἰ ∷ μ ∷ ι ∷ []) "John.10.9"
∷ word (ἡ ∷ []) "John.10.9"
∷ word (θ ∷ ύ ∷ ρ ∷ α ∷ []) "John.10.9"
∷ word (δ ∷ ι ∷ []) "John.10.9"
∷ word (ἐ ∷ μ ∷ ο ∷ ῦ ∷ []) "John.10.9"
∷ word (ἐ ∷ ά ∷ ν ∷ []) "John.10.9"
∷ word (τ ∷ ι ∷ ς ∷ []) "John.10.9"
∷ word (ε ∷ ἰ ∷ σ ∷ έ ∷ ∙λ ∷ θ ∷ ῃ ∷ []) "John.10.9"
∷ word (σ ∷ ω ∷ θ ∷ ή ∷ σ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.10.9"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.10.9"
∷ word (ε ∷ ἰ ∷ σ ∷ ε ∷ ∙λ ∷ ε ∷ ύ ∷ σ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.10.9"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.10.9"
∷ word (ἐ ∷ ξ ∷ ε ∷ ∙λ ∷ ε ∷ ύ ∷ σ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.10.9"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.10.9"
∷ word (ν ∷ ο ∷ μ ∷ ὴ ∷ ν ∷ []) "John.10.9"
∷ word (ε ∷ ὑ ∷ ρ ∷ ή ∷ σ ∷ ε ∷ ι ∷ []) "John.10.9"
∷ word (ὁ ∷ []) "John.10.10"
∷ word (κ ∷ ∙λ ∷ έ ∷ π ∷ τ ∷ η ∷ ς ∷ []) "John.10.10"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.10.10"
∷ word (ἔ ∷ ρ ∷ χ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.10.10"
∷ word (ε ∷ ἰ ∷ []) "John.10.10"
∷ word (μ ∷ ὴ ∷ []) "John.10.10"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.10.10"
∷ word (κ ∷ ∙λ ∷ έ ∷ ψ ∷ ῃ ∷ []) "John.10.10"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.10.10"
∷ word (θ ∷ ύ ∷ σ ∷ ῃ ∷ []) "John.10.10"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.10.10"
∷ word (ἀ ∷ π ∷ ο ∷ ∙λ ∷ έ ∷ σ ∷ ῃ ∷ []) "John.10.10"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.10.10"
∷ word (ἦ ∷ ∙λ ∷ θ ∷ ο ∷ ν ∷ []) "John.10.10"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.10.10"
∷ word (ζ ∷ ω ∷ ὴ ∷ ν ∷ []) "John.10.10"
∷ word (ἔ ∷ χ ∷ ω ∷ σ ∷ ι ∷ ν ∷ []) "John.10.10"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.10.10"
∷ word (π ∷ ε ∷ ρ ∷ ι ∷ σ ∷ σ ∷ ὸ ∷ ν ∷ []) "John.10.10"
∷ word (ἔ ∷ χ ∷ ω ∷ σ ∷ ι ∷ ν ∷ []) "John.10.10"
∷ word (Ἐ ∷ γ ∷ ώ ∷ []) "John.10.11"
∷ word (ε ∷ ἰ ∷ μ ∷ ι ∷ []) "John.10.11"
∷ word (ὁ ∷ []) "John.10.11"
∷ word (π ∷ ο ∷ ι ∷ μ ∷ ὴ ∷ ν ∷ []) "John.10.11"
∷ word (ὁ ∷ []) "John.10.11"
∷ word (κ ∷ α ∷ ∙λ ∷ ό ∷ ς ∷ []) "John.10.11"
∷ word (ὁ ∷ []) "John.10.11"
∷ word (π ∷ ο ∷ ι ∷ μ ∷ ὴ ∷ ν ∷ []) "John.10.11"
∷ word (ὁ ∷ []) "John.10.11"
∷ word (κ ∷ α ∷ ∙λ ∷ ὸ ∷ ς ∷ []) "John.10.11"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.10.11"
∷ word (ψ ∷ υ ∷ χ ∷ ὴ ∷ ν ∷ []) "John.10.11"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.10.11"
∷ word (τ ∷ ί ∷ θ ∷ η ∷ σ ∷ ι ∷ ν ∷ []) "John.10.11"
∷ word (ὑ ∷ π ∷ ὲ ∷ ρ ∷ []) "John.10.11"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.10.11"
∷ word (π ∷ ρ ∷ ο ∷ β ∷ ά ∷ τ ∷ ω ∷ ν ∷ []) "John.10.11"
∷ word (ὁ ∷ []) "John.10.12"
∷ word (μ ∷ ι ∷ σ ∷ θ ∷ ω ∷ τ ∷ ὸ ∷ ς ∷ []) "John.10.12"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.10.12"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.10.12"
∷ word (ὢ ∷ ν ∷ []) "John.10.12"
∷ word (π ∷ ο ∷ ι ∷ μ ∷ ή ∷ ν ∷ []) "John.10.12"
∷ word (ο ∷ ὗ ∷ []) "John.10.12"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.10.12"
∷ word (ἔ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.10.12"
∷ word (τ ∷ ὰ ∷ []) "John.10.12"
∷ word (π ∷ ρ ∷ ό ∷ β ∷ α ∷ τ ∷ α ∷ []) "John.10.12"
∷ word (ἴ ∷ δ ∷ ι ∷ α ∷ []) "John.10.12"
∷ word (θ ∷ ε ∷ ω ∷ ρ ∷ ε ∷ ῖ ∷ []) "John.10.12"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.10.12"
∷ word (∙λ ∷ ύ ∷ κ ∷ ο ∷ ν ∷ []) "John.10.12"
∷ word (ἐ ∷ ρ ∷ χ ∷ ό ∷ μ ∷ ε ∷ ν ∷ ο ∷ ν ∷ []) "John.10.12"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.10.12"
∷ word (ἀ ∷ φ ∷ ί ∷ η ∷ σ ∷ ι ∷ ν ∷ []) "John.10.12"
∷ word (τ ∷ ὰ ∷ []) "John.10.12"
∷ word (π ∷ ρ ∷ ό ∷ β ∷ α ∷ τ ∷ α ∷ []) "John.10.12"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.10.12"
∷ word (φ ∷ ε ∷ ύ ∷ γ ∷ ε ∷ ι ∷ []) "John.10.12"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.10.12"
∷ word (ὁ ∷ []) "John.10.12"
∷ word (∙λ ∷ ύ ∷ κ ∷ ο ∷ ς ∷ []) "John.10.12"
∷ word (ἁ ∷ ρ ∷ π ∷ ά ∷ ζ ∷ ε ∷ ι ∷ []) "John.10.12"
∷ word (α ∷ ὐ ∷ τ ∷ ὰ ∷ []) "John.10.12"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.10.12"
∷ word (σ ∷ κ ∷ ο ∷ ρ ∷ π ∷ ί ∷ ζ ∷ ε ∷ ι ∷ []) "John.10.12"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.10.13"
∷ word (μ ∷ ι ∷ σ ∷ θ ∷ ω ∷ τ ∷ ό ∷ ς ∷ []) "John.10.13"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.10.13"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.10.13"
∷ word (ο ∷ ὐ ∷ []) "John.10.13"
∷ word (μ ∷ έ ∷ ∙λ ∷ ε ∷ ι ∷ []) "John.10.13"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.10.13"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.10.13"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.10.13"
∷ word (π ∷ ρ ∷ ο ∷ β ∷ ά ∷ τ ∷ ω ∷ ν ∷ []) "John.10.13"
∷ word (ἐ ∷ γ ∷ ώ ∷ []) "John.10.14"
∷ word (ε ∷ ἰ ∷ μ ∷ ι ∷ []) "John.10.14"
∷ word (ὁ ∷ []) "John.10.14"
∷ word (π ∷ ο ∷ ι ∷ μ ∷ ὴ ∷ ν ∷ []) "John.10.14"
∷ word (ὁ ∷ []) "John.10.14"
∷ word (κ ∷ α ∷ ∙λ ∷ ό ∷ ς ∷ []) "John.10.14"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.10.14"
∷ word (γ ∷ ι ∷ ν ∷ ώ ∷ σ ∷ κ ∷ ω ∷ []) "John.10.14"
∷ word (τ ∷ ὰ ∷ []) "John.10.14"
∷ word (ἐ ∷ μ ∷ ὰ ∷ []) "John.10.14"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.10.14"
∷ word (γ ∷ ι ∷ ν ∷ ώ ∷ σ ∷ κ ∷ ο ∷ υ ∷ σ ∷ ί ∷ []) "John.10.14"
∷ word (μ ∷ ε ∷ []) "John.10.14"
∷ word (τ ∷ ὰ ∷ []) "John.10.14"
∷ word (ἐ ∷ μ ∷ ά ∷ []) "John.10.14"
∷ word (κ ∷ α ∷ θ ∷ ὼ ∷ ς ∷ []) "John.10.15"
∷ word (γ ∷ ι ∷ ν ∷ ώ ∷ σ ∷ κ ∷ ε ∷ ι ∷ []) "John.10.15"
∷ word (μ ∷ ε ∷ []) "John.10.15"
∷ word (ὁ ∷ []) "John.10.15"
∷ word (π ∷ α ∷ τ ∷ ὴ ∷ ρ ∷ []) "John.10.15"
∷ word (κ ∷ ἀ ∷ γ ∷ ὼ ∷ []) "John.10.15"
∷ word (γ ∷ ι ∷ ν ∷ ώ ∷ σ ∷ κ ∷ ω ∷ []) "John.10.15"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.10.15"
∷ word (π ∷ α ∷ τ ∷ έ ∷ ρ ∷ α ∷ []) "John.10.15"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.10.15"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.10.15"
∷ word (ψ ∷ υ ∷ χ ∷ ή ∷ ν ∷ []) "John.10.15"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.10.15"
∷ word (τ ∷ ί ∷ θ ∷ η ∷ μ ∷ ι ∷ []) "John.10.15"
∷ word (ὑ ∷ π ∷ ὲ ∷ ρ ∷ []) "John.10.15"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.10.15"
∷ word (π ∷ ρ ∷ ο ∷ β ∷ ά ∷ τ ∷ ω ∷ ν ∷ []) "John.10.15"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.10.16"
∷ word (ἄ ∷ ∙λ ∷ ∙λ ∷ α ∷ []) "John.10.16"
∷ word (π ∷ ρ ∷ ό ∷ β ∷ α ∷ τ ∷ α ∷ []) "John.10.16"
∷ word (ἔ ∷ χ ∷ ω ∷ []) "John.10.16"
∷ word (ἃ ∷ []) "John.10.16"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.10.16"
∷ word (ἔ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.10.16"
∷ word (ἐ ∷ κ ∷ []) "John.10.16"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.10.16"
∷ word (α ∷ ὐ ∷ ∙λ ∷ ῆ ∷ ς ∷ []) "John.10.16"
∷ word (τ ∷ α ∷ ύ ∷ τ ∷ η ∷ ς ∷ []) "John.10.16"
∷ word (κ ∷ ἀ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ α ∷ []) "John.10.16"
∷ word (δ ∷ ε ∷ ῖ ∷ []) "John.10.16"
∷ word (μ ∷ ε ∷ []) "John.10.16"
∷ word (ἀ ∷ γ ∷ α ∷ γ ∷ ε ∷ ῖ ∷ ν ∷ []) "John.10.16"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.10.16"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.10.16"
∷ word (φ ∷ ω ∷ ν ∷ ῆ ∷ ς ∷ []) "John.10.16"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.10.16"
∷ word (ἀ ∷ κ ∷ ο ∷ ύ ∷ σ ∷ ο ∷ υ ∷ σ ∷ ι ∷ ν ∷ []) "John.10.16"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.10.16"
∷ word (γ ∷ ε ∷ ν ∷ ή ∷ σ ∷ ο ∷ ν ∷ τ ∷ α ∷ ι ∷ []) "John.10.16"
∷ word (μ ∷ ί ∷ α ∷ []) "John.10.16"
∷ word (π ∷ ο ∷ ί ∷ μ ∷ ν ∷ η ∷ []) "John.10.16"
∷ word (ε ∷ ἷ ∷ ς ∷ []) "John.10.16"
∷ word (π ∷ ο ∷ ι ∷ μ ∷ ή ∷ ν ∷ []) "John.10.16"
∷ word (δ ∷ ι ∷ ὰ ∷ []) "John.10.17"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ό ∷ []) "John.10.17"
∷ word (μ ∷ ε ∷ []) "John.10.17"
∷ word (ὁ ∷ []) "John.10.17"
∷ word (π ∷ α ∷ τ ∷ ὴ ∷ ρ ∷ []) "John.10.17"
∷ word (ἀ ∷ γ ∷ α ∷ π ∷ ᾷ ∷ []) "John.10.17"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.10.17"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.10.17"
∷ word (τ ∷ ί ∷ θ ∷ η ∷ μ ∷ ι ∷ []) "John.10.17"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.10.17"
∷ word (ψ ∷ υ ∷ χ ∷ ή ∷ ν ∷ []) "John.10.17"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.10.17"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.10.17"
∷ word (π ∷ ά ∷ ∙λ ∷ ι ∷ ν ∷ []) "John.10.17"
∷ word (∙λ ∷ ά ∷ β ∷ ω ∷ []) "John.10.17"
∷ word (α ∷ ὐ ∷ τ ∷ ή ∷ ν ∷ []) "John.10.17"
∷ word (ο ∷ ὐ ∷ δ ∷ ε ∷ ὶ ∷ ς ∷ []) "John.10.18"
∷ word (α ∷ ἴ ∷ ρ ∷ ε ∷ ι ∷ []) "John.10.18"
∷ word (α ∷ ὐ ∷ τ ∷ ὴ ∷ ν ∷ []) "John.10.18"
∷ word (ἀ ∷ π ∷ []) "John.10.18"
∷ word (ἐ ∷ μ ∷ ο ∷ ῦ ∷ []) "John.10.18"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ []) "John.10.18"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.10.18"
∷ word (τ ∷ ί ∷ θ ∷ η ∷ μ ∷ ι ∷ []) "John.10.18"
∷ word (α ∷ ὐ ∷ τ ∷ ὴ ∷ ν ∷ []) "John.10.18"
∷ word (ἀ ∷ π ∷ []) "John.10.18"
∷ word (ἐ ∷ μ ∷ α ∷ υ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.10.18"
∷ word (ἐ ∷ ξ ∷ ο ∷ υ ∷ σ ∷ ί ∷ α ∷ ν ∷ []) "John.10.18"
∷ word (ἔ ∷ χ ∷ ω ∷ []) "John.10.18"
∷ word (θ ∷ ε ∷ ῖ ∷ ν ∷ α ∷ ι ∷ []) "John.10.18"
∷ word (α ∷ ὐ ∷ τ ∷ ή ∷ ν ∷ []) "John.10.18"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.10.18"
∷ word (ἐ ∷ ξ ∷ ο ∷ υ ∷ σ ∷ ί ∷ α ∷ ν ∷ []) "John.10.18"
∷ word (ἔ ∷ χ ∷ ω ∷ []) "John.10.18"
∷ word (π ∷ ά ∷ ∙λ ∷ ι ∷ ν ∷ []) "John.10.18"
∷ word (∙λ ∷ α ∷ β ∷ ε ∷ ῖ ∷ ν ∷ []) "John.10.18"
∷ word (α ∷ ὐ ∷ τ ∷ ή ∷ ν ∷ []) "John.10.18"
∷ word (τ ∷ α ∷ ύ ∷ τ ∷ η ∷ ν ∷ []) "John.10.18"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.10.18"
∷ word (ἐ ∷ ν ∷ τ ∷ ο ∷ ∙λ ∷ ὴ ∷ ν ∷ []) "John.10.18"
∷ word (ἔ ∷ ∙λ ∷ α ∷ β ∷ ο ∷ ν ∷ []) "John.10.18"
∷ word (π ∷ α ∷ ρ ∷ ὰ ∷ []) "John.10.18"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.10.18"
∷ word (π ∷ α ∷ τ ∷ ρ ∷ ό ∷ ς ∷ []) "John.10.18"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.10.18"
∷ word (Σ ∷ χ ∷ ί ∷ σ ∷ μ ∷ α ∷ []) "John.10.19"
∷ word (π ∷ ά ∷ ∙λ ∷ ι ∷ ν ∷ []) "John.10.19"
∷ word (ἐ ∷ γ ∷ έ ∷ ν ∷ ε ∷ τ ∷ ο ∷ []) "John.10.19"
∷ word (ἐ ∷ ν ∷ []) "John.10.19"
∷ word (τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.10.19"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ί ∷ ο ∷ ι ∷ ς ∷ []) "John.10.19"
∷ word (δ ∷ ι ∷ ὰ ∷ []) "John.10.19"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.10.19"
∷ word (∙λ ∷ ό ∷ γ ∷ ο ∷ υ ∷ ς ∷ []) "John.10.19"
∷ word (τ ∷ ο ∷ ύ ∷ τ ∷ ο ∷ υ ∷ ς ∷ []) "John.10.19"
∷ word (ἔ ∷ ∙λ ∷ ε ∷ γ ∷ ο ∷ ν ∷ []) "John.10.20"
∷ word (δ ∷ ὲ ∷ []) "John.10.20"
∷ word (π ∷ ο ∷ ∙λ ∷ ∙λ ∷ ο ∷ ὶ ∷ []) "John.10.20"
∷ word (ἐ ∷ ξ ∷ []) "John.10.20"
∷ word (α ∷ ὐ ∷ τ ∷ ῶ ∷ ν ∷ []) "John.10.20"
∷ word (Δ ∷ α ∷ ι ∷ μ ∷ ό ∷ ν ∷ ι ∷ ο ∷ ν ∷ []) "John.10.20"
∷ word (ἔ ∷ χ ∷ ε ∷ ι ∷ []) "John.10.20"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.10.20"
∷ word (μ ∷ α ∷ ί ∷ ν ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.10.20"
∷ word (τ ∷ ί ∷ []) "John.10.20"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.10.20"
∷ word (ἀ ∷ κ ∷ ο ∷ ύ ∷ ε ∷ τ ∷ ε ∷ []) "John.10.20"
∷ word (ἄ ∷ ∙λ ∷ ∙λ ∷ ο ∷ ι ∷ []) "John.10.21"
∷ word (ἔ ∷ ∙λ ∷ ε ∷ γ ∷ ο ∷ ν ∷ []) "John.10.21"
∷ word (Τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.10.21"
∷ word (τ ∷ ὰ ∷ []) "John.10.21"
∷ word (ῥ ∷ ή ∷ μ ∷ α ∷ τ ∷ α ∷ []) "John.10.21"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.10.21"
∷ word (ἔ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.10.21"
∷ word (δ ∷ α ∷ ι ∷ μ ∷ ο ∷ ν ∷ ι ∷ ζ ∷ ο ∷ μ ∷ έ ∷ ν ∷ ο ∷ υ ∷ []) "John.10.21"
∷ word (μ ∷ ὴ ∷ []) "John.10.21"
∷ word (δ ∷ α ∷ ι ∷ μ ∷ ό ∷ ν ∷ ι ∷ ο ∷ ν ∷ []) "John.10.21"
∷ word (δ ∷ ύ ∷ ν ∷ α ∷ τ ∷ α ∷ ι ∷ []) "John.10.21"
∷ word (τ ∷ υ ∷ φ ∷ ∙λ ∷ ῶ ∷ ν ∷ []) "John.10.21"
∷ word (ὀ ∷ φ ∷ θ ∷ α ∷ ∙λ ∷ μ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.10.21"
∷ word (ἀ ∷ ν ∷ ο ∷ ῖ ∷ ξ ∷ α ∷ ι ∷ []) "John.10.21"
∷ word (Ἐ ∷ γ ∷ έ ∷ ν ∷ ε ∷ τ ∷ ο ∷ []) "John.10.22"
∷ word (τ ∷ ό ∷ τ ∷ ε ∷ []) "John.10.22"
∷ word (τ ∷ ὰ ∷ []) "John.10.22"
∷ word (ἐ ∷ γ ∷ κ ∷ α ∷ ί ∷ ν ∷ ι ∷ α ∷ []) "John.10.22"
∷ word (ἐ ∷ ν ∷ []) "John.10.22"
∷ word (τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.10.22"
∷ word (Ἱ ∷ ε ∷ ρ ∷ ο ∷ σ ∷ ο ∷ ∙λ ∷ ύ ∷ μ ∷ ο ∷ ι ∷ ς ∷ []) "John.10.22"
∷ word (χ ∷ ε ∷ ι ∷ μ ∷ ὼ ∷ ν ∷ []) "John.10.22"
∷ word (ἦ ∷ ν ∷ []) "John.10.22"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.10.23"
∷ word (π ∷ ε ∷ ρ ∷ ι ∷ ε ∷ π ∷ ά ∷ τ ∷ ε ∷ ι ∷ []) "John.10.23"
∷ word (ὁ ∷ []) "John.10.23"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.10.23"
∷ word (ἐ ∷ ν ∷ []) "John.10.23"
∷ word (τ ∷ ῷ ∷ []) "John.10.23"
∷ word (ἱ ∷ ε ∷ ρ ∷ ῷ ∷ []) "John.10.23"
∷ word (ἐ ∷ ν ∷ []) "John.10.23"
∷ word (τ ∷ ῇ ∷ []) "John.10.23"
∷ word (σ ∷ τ ∷ ο ∷ ᾷ ∷ []) "John.10.23"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.10.23"
∷ word (Σ ∷ ο ∷ ∙λ ∷ ο ∷ μ ∷ ῶ ∷ ν ∷ ο ∷ ς ∷ []) "John.10.23"
∷ word (ἐ ∷ κ ∷ ύ ∷ κ ∷ ∙λ ∷ ω ∷ σ ∷ α ∷ ν ∷ []) "John.10.24"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.10.24"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.10.24"
∷ word (ο ∷ ἱ ∷ []) "John.10.24"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ῖ ∷ ο ∷ ι ∷ []) "John.10.24"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.10.24"
∷ word (ἔ ∷ ∙λ ∷ ε ∷ γ ∷ ο ∷ ν ∷ []) "John.10.24"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.10.24"
∷ word (Ἕ ∷ ω ∷ ς ∷ []) "John.10.24"
∷ word (π ∷ ό ∷ τ ∷ ε ∷ []) "John.10.24"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.10.24"
∷ word (ψ ∷ υ ∷ χ ∷ ὴ ∷ ν ∷ []) "John.10.24"
∷ word (ἡ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.10.24"
∷ word (α ∷ ἴ ∷ ρ ∷ ε ∷ ι ∷ ς ∷ []) "John.10.24"
∷ word (ε ∷ ἰ ∷ []) "John.10.24"
∷ word (σ ∷ ὺ ∷ []) "John.10.24"
∷ word (ε ∷ ἶ ∷ []) "John.10.24"
∷ word (ὁ ∷ []) "John.10.24"
∷ word (χ ∷ ρ ∷ ι ∷ σ ∷ τ ∷ ό ∷ ς ∷ []) "John.10.24"
∷ word (ε ∷ ἰ ∷ π ∷ ὲ ∷ []) "John.10.24"
∷ word (ἡ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.10.24"
∷ word (π ∷ α ∷ ρ ∷ ρ ∷ η ∷ σ ∷ ί ∷ ᾳ ∷ []) "John.10.24"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.10.25"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.10.25"
∷ word (ὁ ∷ []) "John.10.25"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.10.25"
∷ word (Ε ∷ ἶ ∷ π ∷ ο ∷ ν ∷ []) "John.10.25"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.10.25"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.10.25"
∷ word (ο ∷ ὐ ∷ []) "John.10.25"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ ε ∷ τ ∷ ε ∷ []) "John.10.25"
∷ word (τ ∷ ὰ ∷ []) "John.10.25"
∷ word (ἔ ∷ ρ ∷ γ ∷ α ∷ []) "John.10.25"
∷ word (ἃ ∷ []) "John.10.25"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.10.25"
∷ word (π ∷ ο ∷ ι ∷ ῶ ∷ []) "John.10.25"
∷ word (ἐ ∷ ν ∷ []) "John.10.25"
∷ word (τ ∷ ῷ ∷ []) "John.10.25"
∷ word (ὀ ∷ ν ∷ ό ∷ μ ∷ α ∷ τ ∷ ι ∷ []) "John.10.25"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.10.25"
∷ word (π ∷ α ∷ τ ∷ ρ ∷ ό ∷ ς ∷ []) "John.10.25"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.10.25"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.10.25"
∷ word (μ ∷ α ∷ ρ ∷ τ ∷ υ ∷ ρ ∷ ε ∷ ῖ ∷ []) "John.10.25"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.10.25"
∷ word (ἐ ∷ μ ∷ ο ∷ ῦ ∷ []) "John.10.25"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.10.26"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.10.26"
∷ word (ο ∷ ὐ ∷ []) "John.10.26"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ ε ∷ τ ∷ ε ∷ []) "John.10.26"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.10.26"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.10.26"
∷ word (ἐ ∷ σ ∷ τ ∷ ὲ ∷ []) "John.10.26"
∷ word (ἐ ∷ κ ∷ []) "John.10.26"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.10.26"
∷ word (π ∷ ρ ∷ ο ∷ β ∷ ά ∷ τ ∷ ω ∷ ν ∷ []) "John.10.26"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.10.26"
∷ word (ἐ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.10.26"
∷ word (τ ∷ ὰ ∷ []) "John.10.27"
∷ word (π ∷ ρ ∷ ό ∷ β ∷ α ∷ τ ∷ α ∷ []) "John.10.27"
∷ word (τ ∷ ὰ ∷ []) "John.10.27"
∷ word (ἐ ∷ μ ∷ ὰ ∷ []) "John.10.27"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.10.27"
∷ word (φ ∷ ω ∷ ν ∷ ῆ ∷ ς ∷ []) "John.10.27"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.10.27"
∷ word (ἀ ∷ κ ∷ ο ∷ ύ ∷ ο ∷ υ ∷ σ ∷ ι ∷ ν ∷ []) "John.10.27"
∷ word (κ ∷ ἀ ∷ γ ∷ ὼ ∷ []) "John.10.27"
∷ word (γ ∷ ι ∷ ν ∷ ώ ∷ σ ∷ κ ∷ ω ∷ []) "John.10.27"
∷ word (α ∷ ὐ ∷ τ ∷ ά ∷ []) "John.10.27"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.10.27"
∷ word (ἀ ∷ κ ∷ ο ∷ ∙λ ∷ ο ∷ υ ∷ θ ∷ ο ∷ ῦ ∷ σ ∷ ί ∷ ν ∷ []) "John.10.27"
∷ word (μ ∷ ο ∷ ι ∷ []) "John.10.27"
∷ word (κ ∷ ἀ ∷ γ ∷ ὼ ∷ []) "John.10.28"
∷ word (δ ∷ ί ∷ δ ∷ ω ∷ μ ∷ ι ∷ []) "John.10.28"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.10.28"
∷ word (ζ ∷ ω ∷ ὴ ∷ ν ∷ []) "John.10.28"
∷ word (α ∷ ἰ ∷ ώ ∷ ν ∷ ι ∷ ο ∷ ν ∷ []) "John.10.28"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.10.28"
∷ word (ο ∷ ὐ ∷ []) "John.10.28"
∷ word (μ ∷ ὴ ∷ []) "John.10.28"
∷ word (ἀ ∷ π ∷ ό ∷ ∙λ ∷ ω ∷ ν ∷ τ ∷ α ∷ ι ∷ []) "John.10.28"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.10.28"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.10.28"
∷ word (α ∷ ἰ ∷ ῶ ∷ ν ∷ α ∷ []) "John.10.28"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.10.28"
∷ word (ο ∷ ὐ ∷ χ ∷ []) "John.10.28"
∷ word (ἁ ∷ ρ ∷ π ∷ ά ∷ σ ∷ ε ∷ ι ∷ []) "John.10.28"
∷ word (τ ∷ ι ∷ ς ∷ []) "John.10.28"
∷ word (α ∷ ὐ ∷ τ ∷ ὰ ∷ []) "John.10.28"
∷ word (ἐ ∷ κ ∷ []) "John.10.28"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.10.28"
∷ word (χ ∷ ε ∷ ι ∷ ρ ∷ ό ∷ ς ∷ []) "John.10.28"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.10.28"
∷ word (ὁ ∷ []) "John.10.29"
∷ word (π ∷ α ∷ τ ∷ ή ∷ ρ ∷ []) "John.10.29"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.10.29"
∷ word (ὃ ∷ []) "John.10.29"
∷ word (δ ∷ έ ∷ δ ∷ ω ∷ κ ∷ έ ∷ ν ∷ []) "John.10.29"
∷ word (μ ∷ ο ∷ ι ∷ []) "John.10.29"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ ω ∷ ν ∷ []) "John.10.29"
∷ word (μ ∷ ε ∷ ῖ ∷ ζ ∷ ω ∷ ν ∷ []) "John.10.29"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.10.29"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.10.29"
∷ word (ο ∷ ὐ ∷ δ ∷ ε ∷ ὶ ∷ ς ∷ []) "John.10.29"
∷ word (δ ∷ ύ ∷ ν ∷ α ∷ τ ∷ α ∷ ι ∷ []) "John.10.29"
∷ word (ἁ ∷ ρ ∷ π ∷ ά ∷ ζ ∷ ε ∷ ι ∷ ν ∷ []) "John.10.29"
∷ word (ἐ ∷ κ ∷ []) "John.10.29"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.10.29"
∷ word (χ ∷ ε ∷ ι ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.10.29"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.10.29"
∷ word (π ∷ α ∷ τ ∷ ρ ∷ ό ∷ ς ∷ []) "John.10.29"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.10.30"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.10.30"
∷ word (ὁ ∷ []) "John.10.30"
∷ word (π ∷ α ∷ τ ∷ ὴ ∷ ρ ∷ []) "John.10.30"
∷ word (ἕ ∷ ν ∷ []) "John.10.30"
∷ word (ἐ ∷ σ ∷ μ ∷ ε ∷ ν ∷ []) "John.10.30"
∷ word (Ἐ ∷ β ∷ ά ∷ σ ∷ τ ∷ α ∷ σ ∷ α ∷ ν ∷ []) "John.10.31"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.10.31"
∷ word (π ∷ ά ∷ ∙λ ∷ ι ∷ ν ∷ []) "John.10.31"
∷ word (∙λ ∷ ί ∷ θ ∷ ο ∷ υ ∷ ς ∷ []) "John.10.31"
∷ word (ο ∷ ἱ ∷ []) "John.10.31"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ῖ ∷ ο ∷ ι ∷ []) "John.10.31"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.10.31"
∷ word (∙λ ∷ ι ∷ θ ∷ ά ∷ σ ∷ ω ∷ σ ∷ ι ∷ ν ∷ []) "John.10.31"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.10.31"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.10.32"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.10.32"
∷ word (ὁ ∷ []) "John.10.32"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.10.32"
∷ word (Π ∷ ο ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.10.32"
∷ word (ἔ ∷ ρ ∷ γ ∷ α ∷ []) "John.10.32"
∷ word (κ ∷ α ∷ ∙λ ∷ ὰ ∷ []) "John.10.32"
∷ word (ἔ ∷ δ ∷ ε ∷ ι ∷ ξ ∷ α ∷ []) "John.10.32"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.10.32"
∷ word (ἐ ∷ κ ∷ []) "John.10.32"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.10.32"
∷ word (π ∷ α ∷ τ ∷ ρ ∷ ό ∷ ς ∷ []) "John.10.32"
∷ word (δ ∷ ι ∷ ὰ ∷ []) "John.10.32"
∷ word (π ∷ ο ∷ ῖ ∷ ο ∷ ν ∷ []) "John.10.32"
∷ word (α ∷ ὐ ∷ τ ∷ ῶ ∷ ν ∷ []) "John.10.32"
∷ word (ἔ ∷ ρ ∷ γ ∷ ο ∷ ν ∷ []) "John.10.32"
∷ word (ἐ ∷ μ ∷ ὲ ∷ []) "John.10.32"
∷ word (∙λ ∷ ι ∷ θ ∷ ά ∷ ζ ∷ ε ∷ τ ∷ ε ∷ []) "John.10.32"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.10.33"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.10.33"
∷ word (ο ∷ ἱ ∷ []) "John.10.33"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ῖ ∷ ο ∷ ι ∷ []) "John.10.33"
∷ word (Π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.10.33"
∷ word (κ ∷ α ∷ ∙λ ∷ ο ∷ ῦ ∷ []) "John.10.33"
∷ word (ἔ ∷ ρ ∷ γ ∷ ο ∷ υ ∷ []) "John.10.33"
∷ word (ο ∷ ὐ ∷ []) "John.10.33"
∷ word (∙λ ∷ ι ∷ θ ∷ ά ∷ ζ ∷ ο ∷ μ ∷ έ ∷ ν ∷ []) "John.10.33"
∷ word (σ ∷ ε ∷ []) "John.10.33"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.10.33"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.10.33"
∷ word (β ∷ ∙λ ∷ α ∷ σ ∷ φ ∷ η ∷ μ ∷ ί ∷ α ∷ ς ∷ []) "John.10.33"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.10.33"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.10.33"
∷ word (σ ∷ ὺ ∷ []) "John.10.33"
∷ word (ἄ ∷ ν ∷ θ ∷ ρ ∷ ω ∷ π ∷ ο ∷ ς ∷ []) "John.10.33"
∷ word (ὢ ∷ ν ∷ []) "John.10.33"
∷ word (π ∷ ο ∷ ι ∷ ε ∷ ῖ ∷ ς ∷ []) "John.10.33"
∷ word (σ ∷ ε ∷ α ∷ υ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.10.33"
∷ word (θ ∷ ε ∷ ό ∷ ν ∷ []) "John.10.33"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.10.34"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.10.34"
∷ word (ὁ ∷ []) "John.10.34"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.10.34"
∷ word (Ο ∷ ὐ ∷ κ ∷ []) "John.10.34"
∷ word (ἔ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.10.34"
∷ word (γ ∷ ε ∷ γ ∷ ρ ∷ α ∷ μ ∷ μ ∷ έ ∷ ν ∷ ο ∷ ν ∷ []) "John.10.34"
∷ word (ἐ ∷ ν ∷ []) "John.10.34"
∷ word (τ ∷ ῷ ∷ []) "John.10.34"
∷ word (ν ∷ ό ∷ μ ∷ ῳ ∷ []) "John.10.34"
∷ word (ὑ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.10.34"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.10.34"
∷ word (Ἐ ∷ γ ∷ ὼ ∷ []) "John.10.34"
∷ word (ε ∷ ἶ ∷ π ∷ α ∷ []) "John.10.34"
∷ word (Θ ∷ ε ∷ ο ∷ ί ∷ []) "John.10.34"
∷ word (ἐ ∷ σ ∷ τ ∷ ε ∷ []) "John.10.34"
∷ word (ε ∷ ἰ ∷ []) "John.10.35"
∷ word (ἐ ∷ κ ∷ ε ∷ ί ∷ ν ∷ ο ∷ υ ∷ ς ∷ []) "John.10.35"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.10.35"
∷ word (θ ∷ ε ∷ ο ∷ ὺ ∷ ς ∷ []) "John.10.35"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.10.35"
∷ word (ο ∷ ὓ ∷ ς ∷ []) "John.10.35"
∷ word (ὁ ∷ []) "John.10.35"
∷ word (∙λ ∷ ό ∷ γ ∷ ο ∷ ς ∷ []) "John.10.35"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.10.35"
∷ word (θ ∷ ε ∷ ο ∷ ῦ ∷ []) "John.10.35"
∷ word (ἐ ∷ γ ∷ έ ∷ ν ∷ ε ∷ τ ∷ ο ∷ []) "John.10.35"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.10.35"
∷ word (ο ∷ ὐ ∷ []) "John.10.35"
∷ word (δ ∷ ύ ∷ ν ∷ α ∷ τ ∷ α ∷ ι ∷ []) "John.10.35"
∷ word (∙λ ∷ υ ∷ θ ∷ ῆ ∷ ν ∷ α ∷ ι ∷ []) "John.10.35"
∷ word (ἡ ∷ []) "John.10.35"
∷ word (γ ∷ ρ ∷ α ∷ φ ∷ ή ∷ []) "John.10.35"
∷ word (ὃ ∷ ν ∷ []) "John.10.36"
∷ word (ὁ ∷ []) "John.10.36"
∷ word (π ∷ α ∷ τ ∷ ὴ ∷ ρ ∷ []) "John.10.36"
∷ word (ἡ ∷ γ ∷ ί ∷ α ∷ σ ∷ ε ∷ ν ∷ []) "John.10.36"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.10.36"
∷ word (ἀ ∷ π ∷ έ ∷ σ ∷ τ ∷ ε ∷ ι ∷ ∙λ ∷ ε ∷ ν ∷ []) "John.10.36"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.10.36"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.10.36"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ ν ∷ []) "John.10.36"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.10.36"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ τ ∷ ε ∷ []) "John.10.36"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.10.36"
∷ word (Β ∷ ∙λ ∷ α ∷ σ ∷ φ ∷ η ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.10.36"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.10.36"
∷ word (ε ∷ ἶ ∷ π ∷ ο ∷ ν ∷ []) "John.10.36"
∷ word (Υ ∷ ἱ ∷ ὸ ∷ ς ∷ []) "John.10.36"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.10.36"
∷ word (θ ∷ ε ∷ ο ∷ ῦ ∷ []) "John.10.36"
∷ word (ε ∷ ἰ ∷ μ ∷ ι ∷ []) "John.10.36"
∷ word (ε ∷ ἰ ∷ []) "John.10.37"
∷ word (ο ∷ ὐ ∷ []) "John.10.37"
∷ word (π ∷ ο ∷ ι ∷ ῶ ∷ []) "John.10.37"
∷ word (τ ∷ ὰ ∷ []) "John.10.37"
∷ word (ἔ ∷ ρ ∷ γ ∷ α ∷ []) "John.10.37"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.10.37"
∷ word (π ∷ α ∷ τ ∷ ρ ∷ ό ∷ ς ∷ []) "John.10.37"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.10.37"
∷ word (μ ∷ ὴ ∷ []) "John.10.37"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ ε ∷ τ ∷ έ ∷ []) "John.10.37"
∷ word (μ ∷ ο ∷ ι ∷ []) "John.10.37"
∷ word (ε ∷ ἰ ∷ []) "John.10.38"
∷ word (δ ∷ ὲ ∷ []) "John.10.38"
∷ word (π ∷ ο ∷ ι ∷ ῶ ∷ []) "John.10.38"
∷ word (κ ∷ ἂ ∷ ν ∷ []) "John.10.38"
∷ word (ἐ ∷ μ ∷ ο ∷ ὶ ∷ []) "John.10.38"
∷ word (μ ∷ ὴ ∷ []) "John.10.38"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ η ∷ τ ∷ ε ∷ []) "John.10.38"
∷ word (τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.10.38"
∷ word (ἔ ∷ ρ ∷ γ ∷ ο ∷ ι ∷ ς ∷ []) "John.10.38"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ ε ∷ τ ∷ ε ∷ []) "John.10.38"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.10.38"
∷ word (γ ∷ ν ∷ ῶ ∷ τ ∷ ε ∷ []) "John.10.38"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.10.38"
∷ word (γ ∷ ι ∷ ν ∷ ώ ∷ σ ∷ κ ∷ η ∷ τ ∷ ε ∷ []) "John.10.38"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.10.38"
∷ word (ἐ ∷ ν ∷ []) "John.10.38"
∷ word (ἐ ∷ μ ∷ ο ∷ ὶ ∷ []) "John.10.38"
∷ word (ὁ ∷ []) "John.10.38"
∷ word (π ∷ α ∷ τ ∷ ὴ ∷ ρ ∷ []) "John.10.38"
∷ word (κ ∷ ἀ ∷ γ ∷ ὼ ∷ []) "John.10.38"
∷ word (ἐ ∷ ν ∷ []) "John.10.38"
∷ word (τ ∷ ῷ ∷ []) "John.10.38"
∷ word (π ∷ α ∷ τ ∷ ρ ∷ ί ∷ []) "John.10.38"
∷ word (ἐ ∷ ζ ∷ ή ∷ τ ∷ ο ∷ υ ∷ ν ∷ []) "John.10.39"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.10.39"
∷ word (π ∷ ά ∷ ∙λ ∷ ι ∷ ν ∷ []) "John.10.39"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.10.39"
∷ word (π ∷ ι ∷ ά ∷ σ ∷ α ∷ ι ∷ []) "John.10.39"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.10.39"
∷ word (ἐ ∷ ξ ∷ ῆ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.10.39"
∷ word (ἐ ∷ κ ∷ []) "John.10.39"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.10.39"
∷ word (χ ∷ ε ∷ ι ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.10.39"
∷ word (α ∷ ὐ ∷ τ ∷ ῶ ∷ ν ∷ []) "John.10.39"
∷ word (Κ ∷ α ∷ ὶ ∷ []) "John.10.40"
∷ word (ἀ ∷ π ∷ ῆ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.10.40"
∷ word (π ∷ ά ∷ ∙λ ∷ ι ∷ ν ∷ []) "John.10.40"
∷ word (π ∷ έ ∷ ρ ∷ α ∷ ν ∷ []) "John.10.40"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.10.40"
∷ word (Ἰ ∷ ο ∷ ρ ∷ δ ∷ ά ∷ ν ∷ ο ∷ υ ∷ []) "John.10.40"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.10.40"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.10.40"
∷ word (τ ∷ ό ∷ π ∷ ο ∷ ν ∷ []) "John.10.40"
∷ word (ὅ ∷ π ∷ ο ∷ υ ∷ []) "John.10.40"
∷ word (ἦ ∷ ν ∷ []) "John.10.40"
∷ word (Ἰ ∷ ω ∷ ά ∷ ν ∷ ν ∷ η ∷ ς ∷ []) "John.10.40"
∷ word (τ ∷ ὸ ∷ []) "John.10.40"
∷ word (π ∷ ρ ∷ ῶ ∷ τ ∷ ο ∷ ν ∷ []) "John.10.40"
∷ word (β ∷ α ∷ π ∷ τ ∷ ί ∷ ζ ∷ ω ∷ ν ∷ []) "John.10.40"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.10.40"
∷ word (ἔ ∷ μ ∷ ε ∷ ι ∷ ν ∷ ε ∷ ν ∷ []) "John.10.40"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ []) "John.10.40"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.10.41"
∷ word (π ∷ ο ∷ ∙λ ∷ ∙λ ∷ ο ∷ ὶ ∷ []) "John.10.41"
∷ word (ἦ ∷ ∙λ ∷ θ ∷ ο ∷ ν ∷ []) "John.10.41"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.10.41"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.10.41"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.10.41"
∷ word (ἔ ∷ ∙λ ∷ ε ∷ γ ∷ ο ∷ ν ∷ []) "John.10.41"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.10.41"
∷ word (Ἰ ∷ ω ∷ ά ∷ ν ∷ ν ∷ η ∷ ς ∷ []) "John.10.41"
∷ word (μ ∷ ὲ ∷ ν ∷ []) "John.10.41"
∷ word (σ ∷ η ∷ μ ∷ ε ∷ ῖ ∷ ο ∷ ν ∷ []) "John.10.41"
∷ word (ἐ ∷ π ∷ ο ∷ ί ∷ η ∷ σ ∷ ε ∷ ν ∷ []) "John.10.41"
∷ word (ο ∷ ὐ ∷ δ ∷ έ ∷ ν ∷ []) "John.10.41"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ α ∷ []) "John.10.41"
∷ word (δ ∷ ὲ ∷ []) "John.10.41"
∷ word (ὅ ∷ σ ∷ α ∷ []) "John.10.41"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.10.41"
∷ word (Ἰ ∷ ω ∷ ά ∷ ν ∷ ν ∷ η ∷ ς ∷ []) "John.10.41"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.10.41"
∷ word (τ ∷ ο ∷ ύ ∷ τ ∷ ο ∷ υ ∷ []) "John.10.41"
∷ word (ἀ ∷ ∙λ ∷ η ∷ θ ∷ ῆ ∷ []) "John.10.41"
∷ word (ἦ ∷ ν ∷ []) "John.10.41"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.10.42"
∷ word (π ∷ ο ∷ ∙λ ∷ ∙λ ∷ ο ∷ ὶ ∷ []) "John.10.42"
∷ word (ἐ ∷ π ∷ ί ∷ σ ∷ τ ∷ ε ∷ υ ∷ σ ∷ α ∷ ν ∷ []) "John.10.42"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.10.42"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.10.42"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ []) "John.10.42"
∷ word (Ἦ ∷ ν ∷ []) "John.11.1"
∷ word (δ ∷ έ ∷ []) "John.11.1"
∷ word (τ ∷ ι ∷ ς ∷ []) "John.11.1"
∷ word (ἀ ∷ σ ∷ θ ∷ ε ∷ ν ∷ ῶ ∷ ν ∷ []) "John.11.1"
∷ word (Λ ∷ ά ∷ ζ ∷ α ∷ ρ ∷ ο ∷ ς ∷ []) "John.11.1"
∷ word (ἀ ∷ π ∷ ὸ ∷ []) "John.11.1"
∷ word (Β ∷ η ∷ θ ∷ α ∷ ν ∷ ί ∷ α ∷ ς ∷ []) "John.11.1"
∷ word (ἐ ∷ κ ∷ []) "John.11.1"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.11.1"
∷ word (κ ∷ ώ ∷ μ ∷ η ∷ ς ∷ []) "John.11.1"
∷ word (Μ ∷ α ∷ ρ ∷ ί ∷ α ∷ ς ∷ []) "John.11.1"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.11.1"
∷ word (Μ ∷ ά ∷ ρ ∷ θ ∷ α ∷ ς ∷ []) "John.11.1"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.11.1"
∷ word (ἀ ∷ δ ∷ ε ∷ ∙λ ∷ φ ∷ ῆ ∷ ς ∷ []) "John.11.1"
∷ word (α ∷ ὐ ∷ τ ∷ ῆ ∷ ς ∷ []) "John.11.1"
∷ word (ἦ ∷ ν ∷ []) "John.11.2"
∷ word (δ ∷ ὲ ∷ []) "John.11.2"
∷ word (Μ ∷ α ∷ ρ ∷ ι ∷ ὰ ∷ μ ∷ []) "John.11.2"
∷ word (ἡ ∷ []) "John.11.2"
∷ word (ἀ ∷ ∙λ ∷ ε ∷ ί ∷ ψ ∷ α ∷ σ ∷ α ∷ []) "John.11.2"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.11.2"
∷ word (κ ∷ ύ ∷ ρ ∷ ι ∷ ο ∷ ν ∷ []) "John.11.2"
∷ word (μ ∷ ύ ∷ ρ ∷ ῳ ∷ []) "John.11.2"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.11.2"
∷ word (ἐ ∷ κ ∷ μ ∷ ά ∷ ξ ∷ α ∷ σ ∷ α ∷ []) "John.11.2"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.11.2"
∷ word (π ∷ ό ∷ δ ∷ α ∷ ς ∷ []) "John.11.2"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.11.2"
∷ word (τ ∷ α ∷ ῖ ∷ ς ∷ []) "John.11.2"
∷ word (θ ∷ ρ ∷ ι ∷ ξ ∷ ὶ ∷ ν ∷ []) "John.11.2"
∷ word (α ∷ ὐ ∷ τ ∷ ῆ ∷ ς ∷ []) "John.11.2"
∷ word (ἧ ∷ ς ∷ []) "John.11.2"
∷ word (ὁ ∷ []) "John.11.2"
∷ word (ἀ ∷ δ ∷ ε ∷ ∙λ ∷ φ ∷ ὸ ∷ ς ∷ []) "John.11.2"
∷ word (Λ ∷ ά ∷ ζ ∷ α ∷ ρ ∷ ο ∷ ς ∷ []) "John.11.2"
∷ word (ἠ ∷ σ ∷ θ ∷ έ ∷ ν ∷ ε ∷ ι ∷ []) "John.11.2"
∷ word (ἀ ∷ π ∷ έ ∷ σ ∷ τ ∷ ε ∷ ι ∷ ∙λ ∷ α ∷ ν ∷ []) "John.11.3"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.11.3"
∷ word (α ∷ ἱ ∷ []) "John.11.3"
∷ word (ἀ ∷ δ ∷ ε ∷ ∙λ ∷ φ ∷ α ∷ ὶ ∷ []) "John.11.3"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.11.3"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.11.3"
∷ word (∙λ ∷ έ ∷ γ ∷ ο ∷ υ ∷ σ ∷ α ∷ ι ∷ []) "John.11.3"
∷ word (Κ ∷ ύ ∷ ρ ∷ ι ∷ ε ∷ []) "John.11.3"
∷ word (ἴ ∷ δ ∷ ε ∷ []) "John.11.3"
∷ word (ὃ ∷ ν ∷ []) "John.11.3"
∷ word (φ ∷ ι ∷ ∙λ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.11.3"
∷ word (ἀ ∷ σ ∷ θ ∷ ε ∷ ν ∷ ε ∷ ῖ ∷ []) "John.11.3"
∷ word (ἀ ∷ κ ∷ ο ∷ ύ ∷ σ ∷ α ∷ ς ∷ []) "John.11.4"
∷ word (δ ∷ ὲ ∷ []) "John.11.4"
∷ word (ὁ ∷ []) "John.11.4"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.11.4"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.11.4"
∷ word (Α ∷ ὕ ∷ τ ∷ η ∷ []) "John.11.4"
∷ word (ἡ ∷ []) "John.11.4"
∷ word (ἀ ∷ σ ∷ θ ∷ έ ∷ ν ∷ ε ∷ ι ∷ α ∷ []) "John.11.4"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.11.4"
∷ word (ἔ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.11.4"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.11.4"
∷ word (θ ∷ ά ∷ ν ∷ α ∷ τ ∷ ο ∷ ν ∷ []) "John.11.4"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ []) "John.11.4"
∷ word (ὑ ∷ π ∷ ὲ ∷ ρ ∷ []) "John.11.4"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.11.4"
∷ word (δ ∷ ό ∷ ξ ∷ η ∷ ς ∷ []) "John.11.4"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.11.4"
∷ word (θ ∷ ε ∷ ο ∷ ῦ ∷ []) "John.11.4"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.11.4"
∷ word (δ ∷ ο ∷ ξ ∷ α ∷ σ ∷ θ ∷ ῇ ∷ []) "John.11.4"
∷ word (ὁ ∷ []) "John.11.4"
∷ word (υ ∷ ἱ ∷ ὸ ∷ ς ∷ []) "John.11.4"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.11.4"
∷ word (θ ∷ ε ∷ ο ∷ ῦ ∷ []) "John.11.4"
∷ word (δ ∷ ι ∷ []) "John.11.4"
∷ word (α ∷ ὐ ∷ τ ∷ ῆ ∷ ς ∷ []) "John.11.4"
∷ word (ἠ ∷ γ ∷ ά ∷ π ∷ α ∷ []) "John.11.5"
∷ word (δ ∷ ὲ ∷ []) "John.11.5"
∷ word (ὁ ∷ []) "John.11.5"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.11.5"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.11.5"
∷ word (Μ ∷ ά ∷ ρ ∷ θ ∷ α ∷ ν ∷ []) "John.11.5"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.11.5"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.11.5"
∷ word (ἀ ∷ δ ∷ ε ∷ ∙λ ∷ φ ∷ ὴ ∷ ν ∷ []) "John.11.5"
∷ word (α ∷ ὐ ∷ τ ∷ ῆ ∷ ς ∷ []) "John.11.5"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.11.5"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.11.5"
∷ word (Λ ∷ ά ∷ ζ ∷ α ∷ ρ ∷ ο ∷ ν ∷ []) "John.11.5"
∷ word (ὡ ∷ ς ∷ []) "John.11.6"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.11.6"
∷ word (ἤ ∷ κ ∷ ο ∷ υ ∷ σ ∷ ε ∷ ν ∷ []) "John.11.6"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.11.6"
∷ word (ἀ ∷ σ ∷ θ ∷ ε ∷ ν ∷ ε ∷ ῖ ∷ []) "John.11.6"
∷ word (τ ∷ ό ∷ τ ∷ ε ∷ []) "John.11.6"
∷ word (μ ∷ ὲ ∷ ν ∷ []) "John.11.6"
∷ word (ἔ ∷ μ ∷ ε ∷ ι ∷ ν ∷ ε ∷ ν ∷ []) "John.11.6"
∷ word (ἐ ∷ ν ∷ []) "John.11.6"
∷ word (ᾧ ∷ []) "John.11.6"
∷ word (ἦ ∷ ν ∷ []) "John.11.6"
∷ word (τ ∷ ό ∷ π ∷ ῳ ∷ []) "John.11.6"
∷ word (δ ∷ ύ ∷ ο ∷ []) "John.11.6"
∷ word (ἡ ∷ μ ∷ έ ∷ ρ ∷ α ∷ ς ∷ []) "John.11.6"
∷ word (ἔ ∷ π ∷ ε ∷ ι ∷ τ ∷ α ∷ []) "John.11.7"
∷ word (μ ∷ ε ∷ τ ∷ ὰ ∷ []) "John.11.7"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.11.7"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.11.7"
∷ word (τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.11.7"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ α ∷ ῖ ∷ ς ∷ []) "John.11.7"
∷ word (Ἄ ∷ γ ∷ ω ∷ μ ∷ ε ∷ ν ∷ []) "John.11.7"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.11.7"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.11.7"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ί ∷ α ∷ ν ∷ []) "John.11.7"
∷ word (π ∷ ά ∷ ∙λ ∷ ι ∷ ν ∷ []) "John.11.7"
∷ word (∙λ ∷ έ ∷ γ ∷ ο ∷ υ ∷ σ ∷ ι ∷ ν ∷ []) "John.11.8"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.11.8"
∷ word (ο ∷ ἱ ∷ []) "John.11.8"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ α ∷ ί ∷ []) "John.11.8"
∷ word (Ῥ ∷ α ∷ β ∷ β ∷ ί ∷ []) "John.11.8"
∷ word (ν ∷ ῦ ∷ ν ∷ []) "John.11.8"
∷ word (ἐ ∷ ζ ∷ ή ∷ τ ∷ ο ∷ υ ∷ ν ∷ []) "John.11.8"
∷ word (σ ∷ ε ∷ []) "John.11.8"
∷ word (∙λ ∷ ι ∷ θ ∷ ά ∷ σ ∷ α ∷ ι ∷ []) "John.11.8"
∷ word (ο ∷ ἱ ∷ []) "John.11.8"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ῖ ∷ ο ∷ ι ∷ []) "John.11.8"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.11.8"
∷ word (π ∷ ά ∷ ∙λ ∷ ι ∷ ν ∷ []) "John.11.8"
∷ word (ὑ ∷ π ∷ ά ∷ γ ∷ ε ∷ ι ∷ ς ∷ []) "John.11.8"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ []) "John.11.8"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.11.9"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.11.9"
∷ word (Ο ∷ ὐ ∷ χ ∷ ὶ ∷ []) "John.11.9"
∷ word (δ ∷ ώ ∷ δ ∷ ε ∷ κ ∷ α ∷ []) "John.11.9"
∷ word (ὧ ∷ ρ ∷ α ∷ ί ∷ []) "John.11.9"
∷ word (ε ∷ ἰ ∷ σ ∷ ι ∷ ν ∷ []) "John.11.9"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.11.9"
∷ word (ἡ ∷ μ ∷ έ ∷ ρ ∷ α ∷ ς ∷ []) "John.11.9"
∷ word (ἐ ∷ ά ∷ ν ∷ []) "John.11.9"
∷ word (τ ∷ ι ∷ ς ∷ []) "John.11.9"
∷ word (π ∷ ε ∷ ρ ∷ ι ∷ π ∷ α ∷ τ ∷ ῇ ∷ []) "John.11.9"
∷ word (ἐ ∷ ν ∷ []) "John.11.9"
∷ word (τ ∷ ῇ ∷ []) "John.11.9"
∷ word (ἡ ∷ μ ∷ έ ∷ ρ ∷ ᾳ ∷ []) "John.11.9"
∷ word (ο ∷ ὐ ∷ []) "John.11.9"
∷ word (π ∷ ρ ∷ ο ∷ σ ∷ κ ∷ ό ∷ π ∷ τ ∷ ε ∷ ι ∷ []) "John.11.9"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.11.9"
∷ word (τ ∷ ὸ ∷ []) "John.11.9"
∷ word (φ ∷ ῶ ∷ ς ∷ []) "John.11.9"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.11.9"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ υ ∷ []) "John.11.9"
∷ word (τ ∷ ο ∷ ύ ∷ τ ∷ ο ∷ υ ∷ []) "John.11.9"
∷ word (β ∷ ∙λ ∷ έ ∷ π ∷ ε ∷ ι ∷ []) "John.11.9"
∷ word (ἐ ∷ ὰ ∷ ν ∷ []) "John.11.10"
∷ word (δ ∷ έ ∷ []) "John.11.10"
∷ word (τ ∷ ι ∷ ς ∷ []) "John.11.10"
∷ word (π ∷ ε ∷ ρ ∷ ι ∷ π ∷ α ∷ τ ∷ ῇ ∷ []) "John.11.10"
∷ word (ἐ ∷ ν ∷ []) "John.11.10"
∷ word (τ ∷ ῇ ∷ []) "John.11.10"
∷ word (ν ∷ υ ∷ κ ∷ τ ∷ ί ∷ []) "John.11.10"
∷ word (π ∷ ρ ∷ ο ∷ σ ∷ κ ∷ ό ∷ π ∷ τ ∷ ε ∷ ι ∷ []) "John.11.10"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.11.10"
∷ word (τ ∷ ὸ ∷ []) "John.11.10"
∷ word (φ ∷ ῶ ∷ ς ∷ []) "John.11.10"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.11.10"
∷ word (ἔ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.11.10"
∷ word (ἐ ∷ ν ∷ []) "John.11.10"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.11.10"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.11.11"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.11.11"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.11.11"
∷ word (μ ∷ ε ∷ τ ∷ ὰ ∷ []) "John.11.11"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.11.11"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.11.11"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.11.11"
∷ word (Λ ∷ ά ∷ ζ ∷ α ∷ ρ ∷ ο ∷ ς ∷ []) "John.11.11"
∷ word (ὁ ∷ []) "John.11.11"
∷ word (φ ∷ ί ∷ ∙λ ∷ ο ∷ ς ∷ []) "John.11.11"
∷ word (ἡ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.11.11"
∷ word (κ ∷ ε ∷ κ ∷ ο ∷ ί ∷ μ ∷ η ∷ τ ∷ α ∷ ι ∷ []) "John.11.11"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.11.11"
∷ word (π ∷ ο ∷ ρ ∷ ε ∷ ύ ∷ ο ∷ μ ∷ α ∷ ι ∷ []) "John.11.11"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.11.11"
∷ word (ἐ ∷ ξ ∷ υ ∷ π ∷ ν ∷ ί ∷ σ ∷ ω ∷ []) "John.11.11"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.11.11"
∷ word (ε ∷ ἶ ∷ π ∷ α ∷ ν ∷ []) "John.11.12"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.11.12"
∷ word (ο ∷ ἱ ∷ []) "John.11.12"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ α ∷ ὶ ∷ []) "John.11.12"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.11.12"
∷ word (Κ ∷ ύ ∷ ρ ∷ ι ∷ ε ∷ []) "John.11.12"
∷ word (ε ∷ ἰ ∷ []) "John.11.12"
∷ word (κ ∷ ε ∷ κ ∷ ο ∷ ί ∷ μ ∷ η ∷ τ ∷ α ∷ ι ∷ []) "John.11.12"
∷ word (σ ∷ ω ∷ θ ∷ ή ∷ σ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.11.12"
∷ word (ε ∷ ἰ ∷ ρ ∷ ή ∷ κ ∷ ε ∷ ι ∷ []) "John.11.13"
∷ word (δ ∷ ὲ ∷ []) "John.11.13"
∷ word (ὁ ∷ []) "John.11.13"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.11.13"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.11.13"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.11.13"
∷ word (θ ∷ α ∷ ν ∷ ά ∷ τ ∷ ο ∷ υ ∷ []) "John.11.13"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.11.13"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ο ∷ ι ∷ []) "John.11.13"
∷ word (δ ∷ ὲ ∷ []) "John.11.13"
∷ word (ἔ ∷ δ ∷ ο ∷ ξ ∷ α ∷ ν ∷ []) "John.11.13"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.11.13"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.11.13"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.11.13"
∷ word (κ ∷ ο ∷ ι ∷ μ ∷ ή ∷ σ ∷ ε ∷ ω ∷ ς ∷ []) "John.11.13"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.11.13"
∷ word (ὕ ∷ π ∷ ν ∷ ο ∷ υ ∷ []) "John.11.13"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.11.13"
∷ word (τ ∷ ό ∷ τ ∷ ε ∷ []) "John.11.14"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.11.14"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.11.14"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.11.14"
∷ word (ὁ ∷ []) "John.11.14"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.11.14"
∷ word (π ∷ α ∷ ρ ∷ ρ ∷ η ∷ σ ∷ ί ∷ ᾳ ∷ []) "John.11.14"
∷ word (Λ ∷ ά ∷ ζ ∷ α ∷ ρ ∷ ο ∷ ς ∷ []) "John.11.14"
∷ word (ἀ ∷ π ∷ έ ∷ θ ∷ α ∷ ν ∷ ε ∷ ν ∷ []) "John.11.14"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.11.15"
∷ word (χ ∷ α ∷ ί ∷ ρ ∷ ω ∷ []) "John.11.15"
∷ word (δ ∷ ι ∷ []) "John.11.15"
∷ word (ὑ ∷ μ ∷ ᾶ ∷ ς ∷ []) "John.11.15"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.11.15"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ σ ∷ η ∷ τ ∷ ε ∷ []) "John.11.15"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.11.15"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.11.15"
∷ word (ἤ ∷ μ ∷ η ∷ ν ∷ []) "John.11.15"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ []) "John.11.15"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.11.15"
∷ word (ἄ ∷ γ ∷ ω ∷ μ ∷ ε ∷ ν ∷ []) "John.11.15"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.11.15"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.11.15"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.11.16"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.11.16"
∷ word (Θ ∷ ω ∷ μ ∷ ᾶ ∷ ς ∷ []) "John.11.16"
∷ word (ὁ ∷ []) "John.11.16"
∷ word (∙λ ∷ ε ∷ γ ∷ ό ∷ μ ∷ ε ∷ ν ∷ ο ∷ ς ∷ []) "John.11.16"
∷ word (Δ ∷ ί ∷ δ ∷ υ ∷ μ ∷ ο ∷ ς ∷ []) "John.11.16"
∷ word (τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.11.16"
∷ word (σ ∷ υ ∷ μ ∷ μ ∷ α ∷ θ ∷ η ∷ τ ∷ α ∷ ῖ ∷ ς ∷ []) "John.11.16"
∷ word (Ἄ ∷ γ ∷ ω ∷ μ ∷ ε ∷ ν ∷ []) "John.11.16"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.11.16"
∷ word (ἡ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.11.16"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.11.16"
∷ word (ἀ ∷ π ∷ ο ∷ θ ∷ ά ∷ ν ∷ ω ∷ μ ∷ ε ∷ ν ∷ []) "John.11.16"
∷ word (μ ∷ ε ∷ τ ∷ []) "John.11.16"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.11.16"
∷ word (Ἐ ∷ ∙λ ∷ θ ∷ ὼ ∷ ν ∷ []) "John.11.17"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.11.17"
∷ word (ὁ ∷ []) "John.11.17"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.11.17"
∷ word (ε ∷ ὗ ∷ ρ ∷ ε ∷ ν ∷ []) "John.11.17"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.11.17"
∷ word (τ ∷ έ ∷ σ ∷ σ ∷ α ∷ ρ ∷ α ∷ ς ∷ []) "John.11.17"
∷ word (ἤ ∷ δ ∷ η ∷ []) "John.11.17"
∷ word (ἡ ∷ μ ∷ έ ∷ ρ ∷ α ∷ ς ∷ []) "John.11.17"
∷ word (ἔ ∷ χ ∷ ο ∷ ν ∷ τ ∷ α ∷ []) "John.11.17"
∷ word (ἐ ∷ ν ∷ []) "John.11.17"
∷ word (τ ∷ ῷ ∷ []) "John.11.17"
∷ word (μ ∷ ν ∷ η ∷ μ ∷ ε ∷ ί ∷ ῳ ∷ []) "John.11.17"
∷ word (ἦ ∷ ν ∷ []) "John.11.18"
∷ word (δ ∷ ὲ ∷ []) "John.11.18"
∷ word (ἡ ∷ []) "John.11.18"
∷ word (Β ∷ η ∷ θ ∷ α ∷ ν ∷ ί ∷ α ∷ []) "John.11.18"
∷ word (ἐ ∷ γ ∷ γ ∷ ὺ ∷ ς ∷ []) "John.11.18"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.11.18"
∷ word (Ἱ ∷ ε ∷ ρ ∷ ο ∷ σ ∷ ο ∷ ∙λ ∷ ύ ∷ μ ∷ ω ∷ ν ∷ []) "John.11.18"
∷ word (ὡ ∷ ς ∷ []) "John.11.18"
∷ word (ἀ ∷ π ∷ ὸ ∷ []) "John.11.18"
∷ word (σ ∷ τ ∷ α ∷ δ ∷ ί ∷ ω ∷ ν ∷ []) "John.11.18"
∷ word (δ ∷ ε ∷ κ ∷ α ∷ π ∷ έ ∷ ν ∷ τ ∷ ε ∷ []) "John.11.18"
∷ word (π ∷ ο ∷ ∙λ ∷ ∙λ ∷ ο ∷ ὶ ∷ []) "John.11.19"
∷ word (δ ∷ ὲ ∷ []) "John.11.19"
∷ word (ἐ ∷ κ ∷ []) "John.11.19"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.11.19"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ί ∷ ω ∷ ν ∷ []) "John.11.19"
∷ word (ἐ ∷ ∙λ ∷ η ∷ ∙λ ∷ ύ ∷ θ ∷ ε ∷ ι ∷ σ ∷ α ∷ ν ∷ []) "John.11.19"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.11.19"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.11.19"
∷ word (Μ ∷ ά ∷ ρ ∷ θ ∷ α ∷ ν ∷ []) "John.11.19"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.11.19"
∷ word (Μ ∷ α ∷ ρ ∷ ι ∷ ὰ ∷ μ ∷ []) "John.11.19"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.11.19"
∷ word (π ∷ α ∷ ρ ∷ α ∷ μ ∷ υ ∷ θ ∷ ή ∷ σ ∷ ω ∷ ν ∷ τ ∷ α ∷ ι ∷ []) "John.11.19"
∷ word (α ∷ ὐ ∷ τ ∷ ὰ ∷ ς ∷ []) "John.11.19"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.11.19"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.11.19"
∷ word (ἀ ∷ δ ∷ ε ∷ ∙λ ∷ φ ∷ ο ∷ ῦ ∷ []) "John.11.19"
∷ word (ἡ ∷ []) "John.11.20"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.11.20"
∷ word (Μ ∷ ά ∷ ρ ∷ θ ∷ α ∷ []) "John.11.20"
∷ word (ὡ ∷ ς ∷ []) "John.11.20"
∷ word (ἤ ∷ κ ∷ ο ∷ υ ∷ σ ∷ ε ∷ ν ∷ []) "John.11.20"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.11.20"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.11.20"
∷ word (ἔ ∷ ρ ∷ χ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.11.20"
∷ word (ὑ ∷ π ∷ ή ∷ ν ∷ τ ∷ η ∷ σ ∷ ε ∷ ν ∷ []) "John.11.20"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.11.20"
∷ word (Μ ∷ α ∷ ρ ∷ ί ∷ α ∷ []) "John.11.20"
∷ word (δ ∷ ὲ ∷ []) "John.11.20"
∷ word (ἐ ∷ ν ∷ []) "John.11.20"
∷ word (τ ∷ ῷ ∷ []) "John.11.20"
∷ word (ο ∷ ἴ ∷ κ ∷ ῳ ∷ []) "John.11.20"
∷ word (ἐ ∷ κ ∷ α ∷ θ ∷ έ ∷ ζ ∷ ε ∷ τ ∷ ο ∷ []) "John.11.20"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.11.21"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.11.21"
∷ word (ἡ ∷ []) "John.11.21"
∷ word (Μ ∷ ά ∷ ρ ∷ θ ∷ α ∷ []) "John.11.21"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.11.21"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.11.21"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ν ∷ []) "John.11.21"
∷ word (Κ ∷ ύ ∷ ρ ∷ ι ∷ ε ∷ []) "John.11.21"
∷ word (ε ∷ ἰ ∷ []) "John.11.21"
∷ word (ἦ ∷ ς ∷ []) "John.11.21"
∷ word (ὧ ∷ δ ∷ ε ∷ []) "John.11.21"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.11.21"
∷ word (ἂ ∷ ν ∷ []) "John.11.21"
∷ word (ἀ ∷ π ∷ έ ∷ θ ∷ α ∷ ν ∷ ε ∷ ν ∷ []) "John.11.21"
∷ word (ὁ ∷ []) "John.11.21"
∷ word (ἀ ∷ δ ∷ ε ∷ ∙λ ∷ φ ∷ ό ∷ ς ∷ []) "John.11.21"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.11.21"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.11.22"
∷ word (ν ∷ ῦ ∷ ν ∷ []) "John.11.22"
∷ word (ο ∷ ἶ ∷ δ ∷ α ∷ []) "John.11.22"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.11.22"
∷ word (ὅ ∷ σ ∷ α ∷ []) "John.11.22"
∷ word (ἂ ∷ ν ∷ []) "John.11.22"
∷ word (α ∷ ἰ ∷ τ ∷ ή ∷ σ ∷ ῃ ∷ []) "John.11.22"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.11.22"
∷ word (θ ∷ ε ∷ ὸ ∷ ν ∷ []) "John.11.22"
∷ word (δ ∷ ώ ∷ σ ∷ ε ∷ ι ∷ []) "John.11.22"
∷ word (σ ∷ ο ∷ ι ∷ []) "John.11.22"
∷ word (ὁ ∷ []) "John.11.22"
∷ word (θ ∷ ε ∷ ό ∷ ς ∷ []) "John.11.22"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.11.23"
∷ word (α ∷ ὐ ∷ τ ∷ ῇ ∷ []) "John.11.23"
∷ word (ὁ ∷ []) "John.11.23"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.11.23"
∷ word (Ἀ ∷ ν ∷ α ∷ σ ∷ τ ∷ ή ∷ σ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.11.23"
∷ word (ὁ ∷ []) "John.11.23"
∷ word (ἀ ∷ δ ∷ ε ∷ ∙λ ∷ φ ∷ ό ∷ ς ∷ []) "John.11.23"
∷ word (σ ∷ ο ∷ υ ∷ []) "John.11.23"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.11.24"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.11.24"
∷ word (ἡ ∷ []) "John.11.24"
∷ word (Μ ∷ ά ∷ ρ ∷ θ ∷ α ∷ []) "John.11.24"
∷ word (Ο ∷ ἶ ∷ δ ∷ α ∷ []) "John.11.24"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.11.24"
∷ word (ἀ ∷ ν ∷ α ∷ σ ∷ τ ∷ ή ∷ σ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.11.24"
∷ word (ἐ ∷ ν ∷ []) "John.11.24"
∷ word (τ ∷ ῇ ∷ []) "John.11.24"
∷ word (ἀ ∷ ν ∷ α ∷ σ ∷ τ ∷ ά ∷ σ ∷ ε ∷ ι ∷ []) "John.11.24"
∷ word (ἐ ∷ ν ∷ []) "John.11.24"
∷ word (τ ∷ ῇ ∷ []) "John.11.24"
∷ word (ἐ ∷ σ ∷ χ ∷ ά ∷ τ ∷ ῃ ∷ []) "John.11.24"
∷ word (ἡ ∷ μ ∷ έ ∷ ρ ∷ ᾳ ∷ []) "John.11.24"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.11.25"
∷ word (α ∷ ὐ ∷ τ ∷ ῇ ∷ []) "John.11.25"
∷ word (ὁ ∷ []) "John.11.25"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.11.25"
∷ word (Ἐ ∷ γ ∷ ώ ∷ []) "John.11.25"
∷ word (ε ∷ ἰ ∷ μ ∷ ι ∷ []) "John.11.25"
∷ word (ἡ ∷ []) "John.11.25"
∷ word (ἀ ∷ ν ∷ ά ∷ σ ∷ τ ∷ α ∷ σ ∷ ι ∷ ς ∷ []) "John.11.25"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.11.25"
∷ word (ἡ ∷ []) "John.11.25"
∷ word (ζ ∷ ω ∷ ή ∷ []) "John.11.25"
∷ word (ὁ ∷ []) "John.11.25"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ ω ∷ ν ∷ []) "John.11.25"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.11.25"
∷ word (ἐ ∷ μ ∷ ὲ ∷ []) "John.11.25"
∷ word (κ ∷ ἂ ∷ ν ∷ []) "John.11.25"
∷ word (ἀ ∷ π ∷ ο ∷ θ ∷ ά ∷ ν ∷ ῃ ∷ []) "John.11.25"
∷ word (ζ ∷ ή ∷ σ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.11.25"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.11.26"
∷ word (π ∷ ᾶ ∷ ς ∷ []) "John.11.26"
∷ word (ὁ ∷ []) "John.11.26"
∷ word (ζ ∷ ῶ ∷ ν ∷ []) "John.11.26"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.11.26"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ ω ∷ ν ∷ []) "John.11.26"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.11.26"
∷ word (ἐ ∷ μ ∷ ὲ ∷ []) "John.11.26"
∷ word (ο ∷ ὐ ∷ []) "John.11.26"
∷ word (μ ∷ ὴ ∷ []) "John.11.26"
∷ word (ἀ ∷ π ∷ ο ∷ θ ∷ ά ∷ ν ∷ ῃ ∷ []) "John.11.26"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.11.26"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.11.26"
∷ word (α ∷ ἰ ∷ ῶ ∷ ν ∷ α ∷ []) "John.11.26"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ ε ∷ ι ∷ ς ∷ []) "John.11.26"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.11.26"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.11.27"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.11.27"
∷ word (Ν ∷ α ∷ ί ∷ []) "John.11.27"
∷ word (κ ∷ ύ ∷ ρ ∷ ι ∷ ε ∷ []) "John.11.27"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.11.27"
∷ word (π ∷ ε ∷ π ∷ ί ∷ σ ∷ τ ∷ ε ∷ υ ∷ κ ∷ α ∷ []) "John.11.27"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.11.27"
∷ word (σ ∷ ὺ ∷ []) "John.11.27"
∷ word (ε ∷ ἶ ∷ []) "John.11.27"
∷ word (ὁ ∷ []) "John.11.27"
∷ word (χ ∷ ρ ∷ ι ∷ σ ∷ τ ∷ ὸ ∷ ς ∷ []) "John.11.27"
∷ word (ὁ ∷ []) "John.11.27"
∷ word (υ ∷ ἱ ∷ ὸ ∷ ς ∷ []) "John.11.27"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.11.27"
∷ word (θ ∷ ε ∷ ο ∷ ῦ ∷ []) "John.11.27"
∷ word (ὁ ∷ []) "John.11.27"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.11.27"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.11.27"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ ν ∷ []) "John.11.27"
∷ word (ἐ ∷ ρ ∷ χ ∷ ό ∷ μ ∷ ε ∷ ν ∷ ο ∷ ς ∷ []) "John.11.27"
∷ word (Κ ∷ α ∷ ὶ ∷ []) "John.11.28"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.11.28"
∷ word (ε ∷ ἰ ∷ π ∷ ο ∷ ῦ ∷ σ ∷ α ∷ []) "John.11.28"
∷ word (ἀ ∷ π ∷ ῆ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.11.28"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.11.28"
∷ word (ἐ ∷ φ ∷ ώ ∷ ν ∷ η ∷ σ ∷ ε ∷ ν ∷ []) "John.11.28"
∷ word (Μ ∷ α ∷ ρ ∷ ι ∷ ὰ ∷ μ ∷ []) "John.11.28"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.11.28"
∷ word (ἀ ∷ δ ∷ ε ∷ ∙λ ∷ φ ∷ ὴ ∷ ν ∷ []) "John.11.28"
∷ word (α ∷ ὐ ∷ τ ∷ ῆ ∷ ς ∷ []) "John.11.28"
∷ word (∙λ ∷ ά ∷ θ ∷ ρ ∷ ᾳ ∷ []) "John.11.28"
∷ word (ε ∷ ἰ ∷ π ∷ ο ∷ ῦ ∷ σ ∷ α ∷ []) "John.11.28"
∷ word (Ὁ ∷ []) "John.11.28"
∷ word (δ ∷ ι ∷ δ ∷ ά ∷ σ ∷ κ ∷ α ∷ ∙λ ∷ ο ∷ ς ∷ []) "John.11.28"
∷ word (π ∷ ά ∷ ρ ∷ ε ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.11.28"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.11.28"
∷ word (φ ∷ ω ∷ ν ∷ ε ∷ ῖ ∷ []) "John.11.28"
∷ word (σ ∷ ε ∷ []) "John.11.28"
∷ word (ἐ ∷ κ ∷ ε ∷ ί ∷ ν ∷ η ∷ []) "John.11.29"
∷ word (δ ∷ ὲ ∷ []) "John.11.29"
∷ word (ὡ ∷ ς ∷ []) "John.11.29"
∷ word (ἤ ∷ κ ∷ ο ∷ υ ∷ σ ∷ ε ∷ ν ∷ []) "John.11.29"
∷ word (ἠ ∷ γ ∷ έ ∷ ρ ∷ θ ∷ η ∷ []) "John.11.29"
∷ word (τ ∷ α ∷ χ ∷ ὺ ∷ []) "John.11.29"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.11.29"
∷ word (ἤ ∷ ρ ∷ χ ∷ ε ∷ τ ∷ ο ∷ []) "John.11.29"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.11.29"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.11.29"
∷ word (ο ∷ ὔ ∷ π ∷ ω ∷ []) "John.11.30"
∷ word (δ ∷ ὲ ∷ []) "John.11.30"
∷ word (ἐ ∷ ∙λ ∷ η ∷ ∙λ ∷ ύ ∷ θ ∷ ε ∷ ι ∷ []) "John.11.30"
∷ word (ὁ ∷ []) "John.11.30"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.11.30"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.11.30"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.11.30"
∷ word (κ ∷ ώ ∷ μ ∷ η ∷ ν ∷ []) "John.11.30"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ []) "John.11.30"
∷ word (ἦ ∷ ν ∷ []) "John.11.30"
∷ word (ἔ ∷ τ ∷ ι ∷ []) "John.11.30"
∷ word (ἐ ∷ ν ∷ []) "John.11.30"
∷ word (τ ∷ ῷ ∷ []) "John.11.30"
∷ word (τ ∷ ό ∷ π ∷ ῳ ∷ []) "John.11.30"
∷ word (ὅ ∷ π ∷ ο ∷ υ ∷ []) "John.11.30"
∷ word (ὑ ∷ π ∷ ή ∷ ν ∷ τ ∷ η ∷ σ ∷ ε ∷ ν ∷ []) "John.11.30"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.11.30"
∷ word (ἡ ∷ []) "John.11.30"
∷ word (Μ ∷ ά ∷ ρ ∷ θ ∷ α ∷ []) "John.11.30"
∷ word (ο ∷ ἱ ∷ []) "John.11.31"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.11.31"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ῖ ∷ ο ∷ ι ∷ []) "John.11.31"
∷ word (ο ∷ ἱ ∷ []) "John.11.31"
∷ word (ὄ ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.11.31"
∷ word (μ ∷ ε ∷ τ ∷ []) "John.11.31"
∷ word (α ∷ ὐ ∷ τ ∷ ῆ ∷ ς ∷ []) "John.11.31"
∷ word (ἐ ∷ ν ∷ []) "John.11.31"
∷ word (τ ∷ ῇ ∷ []) "John.11.31"
∷ word (ο ∷ ἰ ∷ κ ∷ ί ∷ ᾳ ∷ []) "John.11.31"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.11.31"
∷ word (π ∷ α ∷ ρ ∷ α ∷ μ ∷ υ ∷ θ ∷ ο ∷ ύ ∷ μ ∷ ε ∷ ν ∷ ο ∷ ι ∷ []) "John.11.31"
∷ word (α ∷ ὐ ∷ τ ∷ ή ∷ ν ∷ []) "John.11.31"
∷ word (ἰ ∷ δ ∷ ό ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.11.31"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.11.31"
∷ word (Μ ∷ α ∷ ρ ∷ ι ∷ ὰ ∷ μ ∷ []) "John.11.31"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.11.31"
∷ word (τ ∷ α ∷ χ ∷ έ ∷ ω ∷ ς ∷ []) "John.11.31"
∷ word (ἀ ∷ ν ∷ έ ∷ σ ∷ τ ∷ η ∷ []) "John.11.31"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.11.31"
∷ word (ἐ ∷ ξ ∷ ῆ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.11.31"
∷ word (ἠ ∷ κ ∷ ο ∷ ∙λ ∷ ο ∷ ύ ∷ θ ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.11.31"
∷ word (α ∷ ὐ ∷ τ ∷ ῇ ∷ []) "John.11.31"
∷ word (δ ∷ ό ∷ ξ ∷ α ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.11.31"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.11.31"
∷ word (ὑ ∷ π ∷ ά ∷ γ ∷ ε ∷ ι ∷ []) "John.11.31"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.11.31"
∷ word (τ ∷ ὸ ∷ []) "John.11.31"
∷ word (μ ∷ ν ∷ η ∷ μ ∷ ε ∷ ῖ ∷ ο ∷ ν ∷ []) "John.11.31"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.11.31"
∷ word (κ ∷ ∙λ ∷ α ∷ ύ ∷ σ ∷ ῃ ∷ []) "John.11.31"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ []) "John.11.31"
∷ word (ἡ ∷ []) "John.11.32"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.11.32"
∷ word (Μ ∷ α ∷ ρ ∷ ι ∷ ὰ ∷ μ ∷ []) "John.11.32"
∷ word (ὡ ∷ ς ∷ []) "John.11.32"
∷ word (ἦ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.11.32"
∷ word (ὅ ∷ π ∷ ο ∷ υ ∷ []) "John.11.32"
∷ word (ἦ ∷ ν ∷ []) "John.11.32"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.11.32"
∷ word (ἰ ∷ δ ∷ ο ∷ ῦ ∷ σ ∷ α ∷ []) "John.11.32"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.11.32"
∷ word (ἔ ∷ π ∷ ε ∷ σ ∷ ε ∷ ν ∷ []) "John.11.32"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.11.32"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.11.32"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.11.32"
∷ word (π ∷ ό ∷ δ ∷ α ∷ ς ∷ []) "John.11.32"
∷ word (∙λ ∷ έ ∷ γ ∷ ο ∷ υ ∷ σ ∷ α ∷ []) "John.11.32"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.11.32"
∷ word (Κ ∷ ύ ∷ ρ ∷ ι ∷ ε ∷ []) "John.11.32"
∷ word (ε ∷ ἰ ∷ []) "John.11.32"
∷ word (ἦ ∷ ς ∷ []) "John.11.32"
∷ word (ὧ ∷ δ ∷ ε ∷ []) "John.11.32"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.11.32"
∷ word (ἄ ∷ ν ∷ []) "John.11.32"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.11.32"
∷ word (ἀ ∷ π ∷ έ ∷ θ ∷ α ∷ ν ∷ ε ∷ ν ∷ []) "John.11.32"
∷ word (ὁ ∷ []) "John.11.32"
∷ word (ἀ ∷ δ ∷ ε ∷ ∙λ ∷ φ ∷ ό ∷ ς ∷ []) "John.11.32"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.11.33"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.11.33"
∷ word (ὡ ∷ ς ∷ []) "John.11.33"
∷ word (ε ∷ ἶ ∷ δ ∷ ε ∷ ν ∷ []) "John.11.33"
∷ word (α ∷ ὐ ∷ τ ∷ ὴ ∷ ν ∷ []) "John.11.33"
∷ word (κ ∷ ∙λ ∷ α ∷ ί ∷ ο ∷ υ ∷ σ ∷ α ∷ ν ∷ []) "John.11.33"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.11.33"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.11.33"
∷ word (σ ∷ υ ∷ ν ∷ ε ∷ ∙λ ∷ θ ∷ ό ∷ ν ∷ τ ∷ α ∷ ς ∷ []) "John.11.33"
∷ word (α ∷ ὐ ∷ τ ∷ ῇ ∷ []) "John.11.33"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ί ∷ ο ∷ υ ∷ ς ∷ []) "John.11.33"
∷ word (κ ∷ ∙λ ∷ α ∷ ί ∷ ο ∷ ν ∷ τ ∷ α ∷ ς ∷ []) "John.11.33"
∷ word (ἐ ∷ ν ∷ ε ∷ β ∷ ρ ∷ ι ∷ μ ∷ ή ∷ σ ∷ α ∷ τ ∷ ο ∷ []) "John.11.33"
∷ word (τ ∷ ῷ ∷ []) "John.11.33"
∷ word (π ∷ ν ∷ ε ∷ ύ ∷ μ ∷ α ∷ τ ∷ ι ∷ []) "John.11.33"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.11.33"
∷ word (ἐ ∷ τ ∷ ά ∷ ρ ∷ α ∷ ξ ∷ ε ∷ ν ∷ []) "John.11.33"
∷ word (ἑ ∷ α ∷ υ ∷ τ ∷ ό ∷ ν ∷ []) "John.11.33"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.11.34"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.11.34"
∷ word (Π ∷ ο ∷ ῦ ∷ []) "John.11.34"
∷ word (τ ∷ ε ∷ θ ∷ ε ∷ ί ∷ κ ∷ α ∷ τ ∷ ε ∷ []) "John.11.34"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.11.34"
∷ word (∙λ ∷ έ ∷ γ ∷ ο ∷ υ ∷ σ ∷ ι ∷ ν ∷ []) "John.11.34"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.11.34"
∷ word (Κ ∷ ύ ∷ ρ ∷ ι ∷ ε ∷ []) "John.11.34"
∷ word (ἔ ∷ ρ ∷ χ ∷ ο ∷ υ ∷ []) "John.11.34"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.11.34"
∷ word (ἴ ∷ δ ∷ ε ∷ []) "John.11.34"
∷ word (ἐ ∷ δ ∷ ά ∷ κ ∷ ρ ∷ υ ∷ σ ∷ ε ∷ ν ∷ []) "John.11.35"
∷ word (ὁ ∷ []) "John.11.35"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.11.35"
∷ word (ἔ ∷ ∙λ ∷ ε ∷ γ ∷ ο ∷ ν ∷ []) "John.11.36"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.11.36"
∷ word (ο ∷ ἱ ∷ []) "John.11.36"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ῖ ∷ ο ∷ ι ∷ []) "John.11.36"
∷ word (Ἴ ∷ δ ∷ ε ∷ []) "John.11.36"
∷ word (π ∷ ῶ ∷ ς ∷ []) "John.11.36"
∷ word (ἐ ∷ φ ∷ ί ∷ ∙λ ∷ ε ∷ ι ∷ []) "John.11.36"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.11.36"
∷ word (τ ∷ ι ∷ ν ∷ ὲ ∷ ς ∷ []) "John.11.37"
∷ word (δ ∷ ὲ ∷ []) "John.11.37"
∷ word (ἐ ∷ ξ ∷ []) "John.11.37"
∷ word (α ∷ ὐ ∷ τ ∷ ῶ ∷ ν ∷ []) "John.11.37"
∷ word (ε ∷ ἶ ∷ π ∷ α ∷ ν ∷ []) "John.11.37"
∷ word (Ο ∷ ὐ ∷ κ ∷ []) "John.11.37"
∷ word (ἐ ∷ δ ∷ ύ ∷ ν ∷ α ∷ τ ∷ ο ∷ []) "John.11.37"
∷ word (ο ∷ ὗ ∷ τ ∷ ο ∷ ς ∷ []) "John.11.37"
∷ word (ὁ ∷ []) "John.11.37"
∷ word (ἀ ∷ ν ∷ ο ∷ ί ∷ ξ ∷ α ∷ ς ∷ []) "John.11.37"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.11.37"
∷ word (ὀ ∷ φ ∷ θ ∷ α ∷ ∙λ ∷ μ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.11.37"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.11.37"
∷ word (τ ∷ υ ∷ φ ∷ ∙λ ∷ ο ∷ ῦ ∷ []) "John.11.37"
∷ word (π ∷ ο ∷ ι ∷ ῆ ∷ σ ∷ α ∷ ι ∷ []) "John.11.37"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.11.37"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.11.37"
∷ word (ο ∷ ὗ ∷ τ ∷ ο ∷ ς ∷ []) "John.11.37"
∷ word (μ ∷ ὴ ∷ []) "John.11.37"
∷ word (ἀ ∷ π ∷ ο ∷ θ ∷ ά ∷ ν ∷ ῃ ∷ []) "John.11.37"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.11.38"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.11.38"
∷ word (π ∷ ά ∷ ∙λ ∷ ι ∷ ν ∷ []) "John.11.38"
∷ word (ἐ ∷ μ ∷ β ∷ ρ ∷ ι ∷ μ ∷ ώ ∷ μ ∷ ε ∷ ν ∷ ο ∷ ς ∷ []) "John.11.38"
∷ word (ἐ ∷ ν ∷ []) "John.11.38"
∷ word (ἑ ∷ α ∷ υ ∷ τ ∷ ῷ ∷ []) "John.11.38"
∷ word (ἔ ∷ ρ ∷ χ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.11.38"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.11.38"
∷ word (τ ∷ ὸ ∷ []) "John.11.38"
∷ word (μ ∷ ν ∷ η ∷ μ ∷ ε ∷ ῖ ∷ ο ∷ ν ∷ []) "John.11.38"
∷ word (ἦ ∷ ν ∷ []) "John.11.38"
∷ word (δ ∷ ὲ ∷ []) "John.11.38"
∷ word (σ ∷ π ∷ ή ∷ ∙λ ∷ α ∷ ι ∷ ο ∷ ν ∷ []) "John.11.38"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.11.38"
∷ word (∙λ ∷ ί ∷ θ ∷ ο ∷ ς ∷ []) "John.11.38"
∷ word (ἐ ∷ π ∷ έ ∷ κ ∷ ε ∷ ι ∷ τ ∷ ο ∷ []) "John.11.38"
∷ word (ἐ ∷ π ∷ []) "John.11.38"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.11.38"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.11.39"
∷ word (ὁ ∷ []) "John.11.39"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.11.39"
∷ word (Ἄ ∷ ρ ∷ α ∷ τ ∷ ε ∷ []) "John.11.39"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.11.39"
∷ word (∙λ ∷ ί ∷ θ ∷ ο ∷ ν ∷ []) "John.11.39"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.11.39"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.11.39"
∷ word (ἡ ∷ []) "John.11.39"
∷ word (ἀ ∷ δ ∷ ε ∷ ∙λ ∷ φ ∷ ὴ ∷ []) "John.11.39"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.11.39"
∷ word (τ ∷ ε ∷ τ ∷ ε ∷ ∙λ ∷ ε ∷ υ ∷ τ ∷ η ∷ κ ∷ ό ∷ τ ∷ ο ∷ ς ∷ []) "John.11.39"
∷ word (Μ ∷ ά ∷ ρ ∷ θ ∷ α ∷ []) "John.11.39"
∷ word (Κ ∷ ύ ∷ ρ ∷ ι ∷ ε ∷ []) "John.11.39"
∷ word (ἤ ∷ δ ∷ η ∷ []) "John.11.39"
∷ word (ὄ ∷ ζ ∷ ε ∷ ι ∷ []) "John.11.39"
∷ word (τ ∷ ε ∷ τ ∷ α ∷ ρ ∷ τ ∷ α ∷ ῖ ∷ ο ∷ ς ∷ []) "John.11.39"
∷ word (γ ∷ ά ∷ ρ ∷ []) "John.11.39"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.11.39"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.11.40"
∷ word (α ∷ ὐ ∷ τ ∷ ῇ ∷ []) "John.11.40"
∷ word (ὁ ∷ []) "John.11.40"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.11.40"
∷ word (Ο ∷ ὐ ∷ κ ∷ []) "John.11.40"
∷ word (ε ∷ ἶ ∷ π ∷ ό ∷ ν ∷ []) "John.11.40"
∷ word (σ ∷ ο ∷ ι ∷ []) "John.11.40"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.11.40"
∷ word (ἐ ∷ ὰ ∷ ν ∷ []) "John.11.40"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ σ ∷ ῃ ∷ ς ∷ []) "John.11.40"
∷ word (ὄ ∷ ψ ∷ ῃ ∷ []) "John.11.40"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.11.40"
∷ word (δ ∷ ό ∷ ξ ∷ α ∷ ν ∷ []) "John.11.40"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.11.40"
∷ word (θ ∷ ε ∷ ο ∷ ῦ ∷ []) "John.11.40"
∷ word (ἦ ∷ ρ ∷ α ∷ ν ∷ []) "John.11.41"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.11.41"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.11.41"
∷ word (∙λ ∷ ί ∷ θ ∷ ο ∷ ν ∷ []) "John.11.41"
∷ word (ὁ ∷ []) "John.11.41"
∷ word (δ ∷ ὲ ∷ []) "John.11.41"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.11.41"
∷ word (ἦ ∷ ρ ∷ ε ∷ ν ∷ []) "John.11.41"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.11.41"
∷ word (ὀ ∷ φ ∷ θ ∷ α ∷ ∙λ ∷ μ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.11.41"
∷ word (ἄ ∷ ν ∷ ω ∷ []) "John.11.41"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.11.41"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.11.41"
∷ word (Π ∷ ά ∷ τ ∷ ε ∷ ρ ∷ []) "John.11.41"
∷ word (ε ∷ ὐ ∷ χ ∷ α ∷ ρ ∷ ι ∷ σ ∷ τ ∷ ῶ ∷ []) "John.11.41"
∷ word (σ ∷ ο ∷ ι ∷ []) "John.11.41"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.11.41"
∷ word (ἤ ∷ κ ∷ ο ∷ υ ∷ σ ∷ ά ∷ ς ∷ []) "John.11.41"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.11.41"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.11.42"
∷ word (δ ∷ ὲ ∷ []) "John.11.42"
∷ word (ᾔ ∷ δ ∷ ε ∷ ι ∷ ν ∷ []) "John.11.42"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.11.42"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ ο ∷ τ ∷ έ ∷ []) "John.11.42"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.11.42"
∷ word (ἀ ∷ κ ∷ ο ∷ ύ ∷ ε ∷ ι ∷ ς ∷ []) "John.11.42"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.11.42"
∷ word (δ ∷ ι ∷ ὰ ∷ []) "John.11.42"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.11.42"
∷ word (ὄ ∷ χ ∷ ∙λ ∷ ο ∷ ν ∷ []) "John.11.42"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.11.42"
∷ word (π ∷ ε ∷ ρ ∷ ι ∷ ε ∷ σ ∷ τ ∷ ῶ ∷ τ ∷ α ∷ []) "John.11.42"
∷ word (ε ∷ ἶ ∷ π ∷ ο ∷ ν ∷ []) "John.11.42"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.11.42"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ σ ∷ ω ∷ σ ∷ ι ∷ ν ∷ []) "John.11.42"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.11.42"
∷ word (σ ∷ ύ ∷ []) "John.11.42"
∷ word (μ ∷ ε ∷ []) "John.11.42"
∷ word (ἀ ∷ π ∷ έ ∷ σ ∷ τ ∷ ε ∷ ι ∷ ∙λ ∷ α ∷ ς ∷ []) "John.11.42"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.11.43"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.11.43"
∷ word (ε ∷ ἰ ∷ π ∷ ὼ ∷ ν ∷ []) "John.11.43"
∷ word (φ ∷ ω ∷ ν ∷ ῇ ∷ []) "John.11.43"
∷ word (μ ∷ ε ∷ γ ∷ ά ∷ ∙λ ∷ ῃ ∷ []) "John.11.43"
∷ word (ἐ ∷ κ ∷ ρ ∷ α ∷ ύ ∷ γ ∷ α ∷ σ ∷ ε ∷ ν ∷ []) "John.11.43"
∷ word (Λ ∷ ά ∷ ζ ∷ α ∷ ρ ∷ ε ∷ []) "John.11.43"
∷ word (δ ∷ ε ∷ ῦ ∷ ρ ∷ ο ∷ []) "John.11.43"
∷ word (ἔ ∷ ξ ∷ ω ∷ []) "John.11.43"
∷ word (ἐ ∷ ξ ∷ ῆ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.11.44"
∷ word (ὁ ∷ []) "John.11.44"
∷ word (τ ∷ ε ∷ θ ∷ ν ∷ η ∷ κ ∷ ὼ ∷ ς ∷ []) "John.11.44"
∷ word (δ ∷ ε ∷ δ ∷ ε ∷ μ ∷ έ ∷ ν ∷ ο ∷ ς ∷ []) "John.11.44"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.11.44"
∷ word (π ∷ ό ∷ δ ∷ α ∷ ς ∷ []) "John.11.44"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.11.44"
∷ word (τ ∷ ὰ ∷ ς ∷ []) "John.11.44"
∷ word (χ ∷ ε ∷ ῖ ∷ ρ ∷ α ∷ ς ∷ []) "John.11.44"
∷ word (κ ∷ ε ∷ ι ∷ ρ ∷ ί ∷ α ∷ ι ∷ ς ∷ []) "John.11.44"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.11.44"
∷ word (ἡ ∷ []) "John.11.44"
∷ word (ὄ ∷ ψ ∷ ι ∷ ς ∷ []) "John.11.44"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.11.44"
∷ word (σ ∷ ο ∷ υ ∷ δ ∷ α ∷ ρ ∷ ί ∷ ῳ ∷ []) "John.11.44"
∷ word (π ∷ ε ∷ ρ ∷ ι ∷ ε ∷ δ ∷ έ ∷ δ ∷ ε ∷ τ ∷ ο ∷ []) "John.11.44"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.11.44"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.11.44"
∷ word (ὁ ∷ []) "John.11.44"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.11.44"
∷ word (Λ ∷ ύ ∷ σ ∷ α ∷ τ ∷ ε ∷ []) "John.11.44"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.11.44"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.11.44"
∷ word (ἄ ∷ φ ∷ ε ∷ τ ∷ ε ∷ []) "John.11.44"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.11.44"
∷ word (ὑ ∷ π ∷ ά ∷ γ ∷ ε ∷ ι ∷ ν ∷ []) "John.11.44"
∷ word (Π ∷ ο ∷ ∙λ ∷ ∙λ ∷ ο ∷ ὶ ∷ []) "John.11.45"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.11.45"
∷ word (ἐ ∷ κ ∷ []) "John.11.45"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.11.45"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ί ∷ ω ∷ ν ∷ []) "John.11.45"
∷ word (ο ∷ ἱ ∷ []) "John.11.45"
∷ word (ἐ ∷ ∙λ ∷ θ ∷ ό ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.11.45"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.11.45"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.11.45"
∷ word (Μ ∷ α ∷ ρ ∷ ι ∷ ὰ ∷ μ ∷ []) "John.11.45"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.11.45"
∷ word (θ ∷ ε ∷ α ∷ σ ∷ ά ∷ μ ∷ ε ∷ ν ∷ ο ∷ ι ∷ []) "John.11.45"
∷ word (ἃ ∷ []) "John.11.45"
∷ word (ἐ ∷ π ∷ ο ∷ ί ∷ η ∷ σ ∷ ε ∷ ν ∷ []) "John.11.45"
∷ word (ἐ ∷ π ∷ ί ∷ σ ∷ τ ∷ ε ∷ υ ∷ σ ∷ α ∷ ν ∷ []) "John.11.45"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.11.45"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.11.45"
∷ word (τ ∷ ι ∷ ν ∷ ὲ ∷ ς ∷ []) "John.11.46"
∷ word (δ ∷ ὲ ∷ []) "John.11.46"
∷ word (ἐ ∷ ξ ∷ []) "John.11.46"
∷ word (α ∷ ὐ ∷ τ ∷ ῶ ∷ ν ∷ []) "John.11.46"
∷ word (ἀ ∷ π ∷ ῆ ∷ ∙λ ∷ θ ∷ ο ∷ ν ∷ []) "John.11.46"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.11.46"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.11.46"
∷ word (Φ ∷ α ∷ ρ ∷ ι ∷ σ ∷ α ∷ ί ∷ ο ∷ υ ∷ ς ∷ []) "John.11.46"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.11.46"
∷ word (ε ∷ ἶ ∷ π ∷ α ∷ ν ∷ []) "John.11.46"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.11.46"
∷ word (ἃ ∷ []) "John.11.46"
∷ word (ἐ ∷ π ∷ ο ∷ ί ∷ η ∷ σ ∷ ε ∷ ν ∷ []) "John.11.46"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.11.46"
∷ word (σ ∷ υ ∷ ν ∷ ή ∷ γ ∷ α ∷ γ ∷ ο ∷ ν ∷ []) "John.11.47"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.11.47"
∷ word (ο ∷ ἱ ∷ []) "John.11.47"
∷ word (ἀ ∷ ρ ∷ χ ∷ ι ∷ ε ∷ ρ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.11.47"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.11.47"
∷ word (ο ∷ ἱ ∷ []) "John.11.47"
∷ word (Φ ∷ α ∷ ρ ∷ ι ∷ σ ∷ α ∷ ῖ ∷ ο ∷ ι ∷ []) "John.11.47"
∷ word (σ ∷ υ ∷ ν ∷ έ ∷ δ ∷ ρ ∷ ι ∷ ο ∷ ν ∷ []) "John.11.47"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.11.47"
∷ word (ἔ ∷ ∙λ ∷ ε ∷ γ ∷ ο ∷ ν ∷ []) "John.11.47"
∷ word (Τ ∷ ί ∷ []) "John.11.47"
∷ word (π ∷ ο ∷ ι ∷ ο ∷ ῦ ∷ μ ∷ ε ∷ ν ∷ []) "John.11.47"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.11.47"
∷ word (ο ∷ ὗ ∷ τ ∷ ο ∷ ς ∷ []) "John.11.47"
∷ word (ὁ ∷ []) "John.11.47"
∷ word (ἄ ∷ ν ∷ θ ∷ ρ ∷ ω ∷ π ∷ ο ∷ ς ∷ []) "John.11.47"
∷ word (π ∷ ο ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.11.47"
∷ word (π ∷ ο ∷ ι ∷ ε ∷ ῖ ∷ []) "John.11.47"
∷ word (σ ∷ η ∷ μ ∷ ε ∷ ῖ ∷ α ∷ []) "John.11.47"
∷ word (ἐ ∷ ὰ ∷ ν ∷ []) "John.11.48"
∷ word (ἀ ∷ φ ∷ ῶ ∷ μ ∷ ε ∷ ν ∷ []) "John.11.48"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.11.48"
∷ word (ο ∷ ὕ ∷ τ ∷ ω ∷ ς ∷ []) "John.11.48"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.11.48"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ σ ∷ ο ∷ υ ∷ σ ∷ ι ∷ ν ∷ []) "John.11.48"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.11.48"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.11.48"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.11.48"
∷ word (ἐ ∷ ∙λ ∷ ε ∷ ύ ∷ σ ∷ ο ∷ ν ∷ τ ∷ α ∷ ι ∷ []) "John.11.48"
∷ word (ο ∷ ἱ ∷ []) "John.11.48"
∷ word (Ῥ ∷ ω ∷ μ ∷ α ∷ ῖ ∷ ο ∷ ι ∷ []) "John.11.48"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.11.48"
∷ word (ἀ ∷ ρ ∷ ο ∷ ῦ ∷ σ ∷ ι ∷ ν ∷ []) "John.11.48"
∷ word (ἡ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.11.48"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.11.48"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.11.48"
∷ word (τ ∷ ό ∷ π ∷ ο ∷ ν ∷ []) "John.11.48"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.11.48"
∷ word (τ ∷ ὸ ∷ []) "John.11.48"
∷ word (ἔ ∷ θ ∷ ν ∷ ο ∷ ς ∷ []) "John.11.48"
∷ word (ε ∷ ἷ ∷ ς ∷ []) "John.11.49"
∷ word (δ ∷ έ ∷ []) "John.11.49"
∷ word (τ ∷ ι ∷ ς ∷ []) "John.11.49"
∷ word (ἐ ∷ ξ ∷ []) "John.11.49"
∷ word (α ∷ ὐ ∷ τ ∷ ῶ ∷ ν ∷ []) "John.11.49"
∷ word (Κ ∷ α ∷ ϊ ∷ ά ∷ φ ∷ α ∷ ς ∷ []) "John.11.49"
∷ word (ἀ ∷ ρ ∷ χ ∷ ι ∷ ε ∷ ρ ∷ ε ∷ ὺ ∷ ς ∷ []) "John.11.49"
∷ word (ὢ ∷ ν ∷ []) "John.11.49"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.11.49"
∷ word (ἐ ∷ ν ∷ ι ∷ α ∷ υ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.11.49"
∷ word (ἐ ∷ κ ∷ ε ∷ ί ∷ ν ∷ ο ∷ υ ∷ []) "John.11.49"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.11.49"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.11.49"
∷ word (Ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.11.49"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.11.49"
∷ word (ο ∷ ἴ ∷ δ ∷ α ∷ τ ∷ ε ∷ []) "John.11.49"
∷ word (ο ∷ ὐ ∷ δ ∷ έ ∷ ν ∷ []) "John.11.49"
∷ word (ο ∷ ὐ ∷ δ ∷ ὲ ∷ []) "John.11.50"
∷ word (∙λ ∷ ο ∷ γ ∷ ί ∷ ζ ∷ ε ∷ σ ∷ θ ∷ ε ∷ []) "John.11.50"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.11.50"
∷ word (σ ∷ υ ∷ μ ∷ φ ∷ έ ∷ ρ ∷ ε ∷ ι ∷ []) "John.11.50"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.11.50"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.11.50"
∷ word (ε ∷ ἷ ∷ ς ∷ []) "John.11.50"
∷ word (ἄ ∷ ν ∷ θ ∷ ρ ∷ ω ∷ π ∷ ο ∷ ς ∷ []) "John.11.50"
∷ word (ἀ ∷ π ∷ ο ∷ θ ∷ ά ∷ ν ∷ ῃ ∷ []) "John.11.50"
∷ word (ὑ ∷ π ∷ ὲ ∷ ρ ∷ []) "John.11.50"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.11.50"
∷ word (∙λ ∷ α ∷ ο ∷ ῦ ∷ []) "John.11.50"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.11.50"
∷ word (μ ∷ ὴ ∷ []) "John.11.50"
∷ word (ὅ ∷ ∙λ ∷ ο ∷ ν ∷ []) "John.11.50"
∷ word (τ ∷ ὸ ∷ []) "John.11.50"
∷ word (ἔ ∷ θ ∷ ν ∷ ο ∷ ς ∷ []) "John.11.50"
∷ word (ἀ ∷ π ∷ ό ∷ ∙λ ∷ η ∷ τ ∷ α ∷ ι ∷ []) "John.11.50"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.11.51"
∷ word (δ ∷ ὲ ∷ []) "John.11.51"
∷ word (ἀ ∷ φ ∷ []) "John.11.51"
∷ word (ἑ ∷ α ∷ υ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.11.51"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.11.51"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.11.51"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.11.51"
∷ word (ἀ ∷ ρ ∷ χ ∷ ι ∷ ε ∷ ρ ∷ ε ∷ ὺ ∷ ς ∷ []) "John.11.51"
∷ word (ὢ ∷ ν ∷ []) "John.11.51"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.11.51"
∷ word (ἐ ∷ ν ∷ ι ∷ α ∷ υ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.11.51"
∷ word (ἐ ∷ κ ∷ ε ∷ ί ∷ ν ∷ ο ∷ υ ∷ []) "John.11.51"
∷ word (ἐ ∷ π ∷ ρ ∷ ο ∷ φ ∷ ή ∷ τ ∷ ε ∷ υ ∷ σ ∷ ε ∷ ν ∷ []) "John.11.51"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.11.51"
∷ word (ἔ ∷ μ ∷ ε ∷ ∙λ ∷ ∙λ ∷ ε ∷ ν ∷ []) "John.11.51"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.11.51"
∷ word (ἀ ∷ π ∷ ο ∷ θ ∷ ν ∷ ῄ ∷ σ ∷ κ ∷ ε ∷ ι ∷ ν ∷ []) "John.11.51"
∷ word (ὑ ∷ π ∷ ὲ ∷ ρ ∷ []) "John.11.51"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.11.51"
∷ word (ἔ ∷ θ ∷ ν ∷ ο ∷ υ ∷ ς ∷ []) "John.11.51"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.11.52"
∷ word (ο ∷ ὐ ∷ χ ∷ []) "John.11.52"
∷ word (ὑ ∷ π ∷ ὲ ∷ ρ ∷ []) "John.11.52"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.11.52"
∷ word (ἔ ∷ θ ∷ ν ∷ ο ∷ υ ∷ ς ∷ []) "John.11.52"
∷ word (μ ∷ ό ∷ ν ∷ ο ∷ ν ∷ []) "John.11.52"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ []) "John.11.52"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.11.52"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.11.52"
∷ word (τ ∷ ὰ ∷ []) "John.11.52"
∷ word (τ ∷ έ ∷ κ ∷ ν ∷ α ∷ []) "John.11.52"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.11.52"
∷ word (θ ∷ ε ∷ ο ∷ ῦ ∷ []) "John.11.52"
∷ word (τ ∷ ὰ ∷ []) "John.11.52"
∷ word (δ ∷ ι ∷ ε ∷ σ ∷ κ ∷ ο ∷ ρ ∷ π ∷ ι ∷ σ ∷ μ ∷ έ ∷ ν ∷ α ∷ []) "John.11.52"
∷ word (σ ∷ υ ∷ ν ∷ α ∷ γ ∷ ά ∷ γ ∷ ῃ ∷ []) "John.11.52"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.11.52"
∷ word (ἕ ∷ ν ∷ []) "John.11.52"
∷ word (ἀ ∷ π ∷ []) "John.11.53"
∷ word (ἐ ∷ κ ∷ ε ∷ ί ∷ ν ∷ η ∷ ς ∷ []) "John.11.53"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.11.53"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.11.53"
∷ word (ἡ ∷ μ ∷ έ ∷ ρ ∷ α ∷ ς ∷ []) "John.11.53"
∷ word (ἐ ∷ β ∷ ο ∷ υ ∷ ∙λ ∷ ε ∷ ύ ∷ σ ∷ α ∷ ν ∷ τ ∷ ο ∷ []) "John.11.53"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.11.53"
∷ word (ἀ ∷ π ∷ ο ∷ κ ∷ τ ∷ ε ∷ ί ∷ ν ∷ ω ∷ σ ∷ ι ∷ ν ∷ []) "John.11.53"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.11.53"
∷ word (Ὁ ∷ []) "John.11.54"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.11.54"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.11.54"
∷ word (ο ∷ ὐ ∷ κ ∷ έ ∷ τ ∷ ι ∷ []) "John.11.54"
∷ word (π ∷ α ∷ ρ ∷ ρ ∷ η ∷ σ ∷ ί ∷ ᾳ ∷ []) "John.11.54"
∷ word (π ∷ ε ∷ ρ ∷ ι ∷ ε ∷ π ∷ ά ∷ τ ∷ ε ∷ ι ∷ []) "John.11.54"
∷ word (ἐ ∷ ν ∷ []) "John.11.54"
∷ word (τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.11.54"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ί ∷ ο ∷ ι ∷ ς ∷ []) "John.11.54"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.11.54"
∷ word (ἀ ∷ π ∷ ῆ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.11.54"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ θ ∷ ε ∷ ν ∷ []) "John.11.54"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.11.54"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.11.54"
∷ word (χ ∷ ώ ∷ ρ ∷ α ∷ ν ∷ []) "John.11.54"
∷ word (ἐ ∷ γ ∷ γ ∷ ὺ ∷ ς ∷ []) "John.11.54"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.11.54"
∷ word (ἐ ∷ ρ ∷ ή ∷ μ ∷ ο ∷ υ ∷ []) "John.11.54"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.11.54"
∷ word (Ἐ ∷ φ ∷ ρ ∷ α ∷ ὶ ∷ μ ∷ []) "John.11.54"
∷ word (∙λ ∷ ε ∷ γ ∷ ο ∷ μ ∷ έ ∷ ν ∷ η ∷ ν ∷ []) "John.11.54"
∷ word (π ∷ ό ∷ ∙λ ∷ ι ∷ ν ∷ []) "John.11.54"
∷ word (κ ∷ ἀ ∷ κ ∷ ε ∷ ῖ ∷ []) "John.11.54"
∷ word (ἔ ∷ μ ∷ ε ∷ ι ∷ ν ∷ ε ∷ ν ∷ []) "John.11.54"
∷ word (μ ∷ ε ∷ τ ∷ ὰ ∷ []) "John.11.54"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.11.54"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ ῶ ∷ ν ∷ []) "John.11.54"
∷ word (Ἦ ∷ ν ∷ []) "John.11.55"
∷ word (δ ∷ ὲ ∷ []) "John.11.55"
∷ word (ἐ ∷ γ ∷ γ ∷ ὺ ∷ ς ∷ []) "John.11.55"
∷ word (τ ∷ ὸ ∷ []) "John.11.55"
∷ word (π ∷ ά ∷ σ ∷ χ ∷ α ∷ []) "John.11.55"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.11.55"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ί ∷ ω ∷ ν ∷ []) "John.11.55"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.11.55"
∷ word (ἀ ∷ ν ∷ έ ∷ β ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.11.55"
∷ word (π ∷ ο ∷ ∙λ ∷ ∙λ ∷ ο ∷ ὶ ∷ []) "John.11.55"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.11.55"
∷ word (Ἱ ∷ ε ∷ ρ ∷ ο ∷ σ ∷ ό ∷ ∙λ ∷ υ ∷ μ ∷ α ∷ []) "John.11.55"
∷ word (ἐ ∷ κ ∷ []) "John.11.55"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.11.55"
∷ word (χ ∷ ώ ∷ ρ ∷ α ∷ ς ∷ []) "John.11.55"
∷ word (π ∷ ρ ∷ ὸ ∷ []) "John.11.55"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.11.55"
∷ word (π ∷ ά ∷ σ ∷ χ ∷ α ∷ []) "John.11.55"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.11.55"
∷ word (ἁ ∷ γ ∷ ν ∷ ί ∷ σ ∷ ω ∷ σ ∷ ι ∷ ν ∷ []) "John.11.55"
∷ word (ἑ ∷ α ∷ υ ∷ τ ∷ ο ∷ ύ ∷ ς ∷ []) "John.11.55"
∷ word (ἐ ∷ ζ ∷ ή ∷ τ ∷ ο ∷ υ ∷ ν ∷ []) "John.11.56"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.11.56"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.11.56"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ν ∷ []) "John.11.56"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.11.56"
∷ word (ἔ ∷ ∙λ ∷ ε ∷ γ ∷ ο ∷ ν ∷ []) "John.11.56"
∷ word (μ ∷ ε ∷ τ ∷ []) "John.11.56"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ή ∷ ∙λ ∷ ω ∷ ν ∷ []) "John.11.56"
∷ word (ἐ ∷ ν ∷ []) "John.11.56"
∷ word (τ ∷ ῷ ∷ []) "John.11.56"
∷ word (ἱ ∷ ε ∷ ρ ∷ ῷ ∷ []) "John.11.56"
∷ word (ἑ ∷ σ ∷ τ ∷ η ∷ κ ∷ ό ∷ τ ∷ ε ∷ ς ∷ []) "John.11.56"
∷ word (Τ ∷ ί ∷ []) "John.11.56"
∷ word (δ ∷ ο ∷ κ ∷ ε ∷ ῖ ∷ []) "John.11.56"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.11.56"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.11.56"
∷ word (ο ∷ ὐ ∷ []) "John.11.56"
∷ word (μ ∷ ὴ ∷ []) "John.11.56"
∷ word (ἔ ∷ ∙λ ∷ θ ∷ ῃ ∷ []) "John.11.56"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.11.56"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.11.56"
∷ word (ἑ ∷ ο ∷ ρ ∷ τ ∷ ή ∷ ν ∷ []) "John.11.56"
∷ word (δ ∷ ε ∷ δ ∷ ώ ∷ κ ∷ ε ∷ ι ∷ σ ∷ α ∷ ν ∷ []) "John.11.57"
∷ word (δ ∷ ὲ ∷ []) "John.11.57"
∷ word (ο ∷ ἱ ∷ []) "John.11.57"
∷ word (ἀ ∷ ρ ∷ χ ∷ ι ∷ ε ∷ ρ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.11.57"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.11.57"
∷ word (ο ∷ ἱ ∷ []) "John.11.57"
∷ word (Φ ∷ α ∷ ρ ∷ ι ∷ σ ∷ α ∷ ῖ ∷ ο ∷ ι ∷ []) "John.11.57"
∷ word (ἐ ∷ ν ∷ τ ∷ ο ∷ ∙λ ∷ ὰ ∷ ς ∷ []) "John.11.57"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.11.57"
∷ word (ἐ ∷ ά ∷ ν ∷ []) "John.11.57"
∷ word (τ ∷ ι ∷ ς ∷ []) "John.11.57"
∷ word (γ ∷ ν ∷ ῷ ∷ []) "John.11.57"
∷ word (π ∷ ο ∷ ῦ ∷ []) "John.11.57"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.11.57"
∷ word (μ ∷ η ∷ ν ∷ ύ ∷ σ ∷ ῃ ∷ []) "John.11.57"
∷ word (ὅ ∷ π ∷ ω ∷ ς ∷ []) "John.11.57"
∷ word (π ∷ ι ∷ ά ∷ σ ∷ ω ∷ σ ∷ ι ∷ ν ∷ []) "John.11.57"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.11.57"
∷ word (Ὁ ∷ []) "John.12.1"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.12.1"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.12.1"
∷ word (π ∷ ρ ∷ ὸ ∷ []) "John.12.1"
∷ word (ἓ ∷ ξ ∷ []) "John.12.1"
∷ word (ἡ ∷ μ ∷ ε ∷ ρ ∷ ῶ ∷ ν ∷ []) "John.12.1"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.12.1"
∷ word (π ∷ ά ∷ σ ∷ χ ∷ α ∷ []) "John.12.1"
∷ word (ἦ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.12.1"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.12.1"
∷ word (Β ∷ η ∷ θ ∷ α ∷ ν ∷ ί ∷ α ∷ ν ∷ []) "John.12.1"
∷ word (ὅ ∷ π ∷ ο ∷ υ ∷ []) "John.12.1"
∷ word (ἦ ∷ ν ∷ []) "John.12.1"
∷ word (Λ ∷ ά ∷ ζ ∷ α ∷ ρ ∷ ο ∷ ς ∷ []) "John.12.1"
∷ word (ὃ ∷ ν ∷ []) "John.12.1"
∷ word (ἤ ∷ γ ∷ ε ∷ ι ∷ ρ ∷ ε ∷ ν ∷ []) "John.12.1"
∷ word (ἐ ∷ κ ∷ []) "John.12.1"
∷ word (ν ∷ ε ∷ κ ∷ ρ ∷ ῶ ∷ ν ∷ []) "John.12.1"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.12.1"
∷ word (ἐ ∷ π ∷ ο ∷ ί ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.12.2"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.12.2"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.12.2"
∷ word (δ ∷ ε ∷ ῖ ∷ π ∷ ν ∷ ο ∷ ν ∷ []) "John.12.2"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ []) "John.12.2"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.12.2"
∷ word (ἡ ∷ []) "John.12.2"
∷ word (Μ ∷ ά ∷ ρ ∷ θ ∷ α ∷ []) "John.12.2"
∷ word (δ ∷ ι ∷ η ∷ κ ∷ ό ∷ ν ∷ ε ∷ ι ∷ []) "John.12.2"
∷ word (ὁ ∷ []) "John.12.2"
∷ word (δ ∷ ὲ ∷ []) "John.12.2"
∷ word (Λ ∷ ά ∷ ζ ∷ α ∷ ρ ∷ ο ∷ ς ∷ []) "John.12.2"
∷ word (ε ∷ ἷ ∷ ς ∷ []) "John.12.2"
∷ word (ἦ ∷ ν ∷ []) "John.12.2"
∷ word (ἐ ∷ κ ∷ []) "John.12.2"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.12.2"
∷ word (ἀ ∷ ν ∷ α ∷ κ ∷ ε ∷ ι ∷ μ ∷ έ ∷ ν ∷ ω ∷ ν ∷ []) "John.12.2"
∷ word (σ ∷ ὺ ∷ ν ∷ []) "John.12.2"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.12.2"
∷ word (ἡ ∷ []) "John.12.3"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.12.3"
∷ word (Μ ∷ α ∷ ρ ∷ ι ∷ ὰ ∷ μ ∷ []) "John.12.3"
∷ word (∙λ ∷ α ∷ β ∷ ο ∷ ῦ ∷ σ ∷ α ∷ []) "John.12.3"
∷ word (∙λ ∷ ί ∷ τ ∷ ρ ∷ α ∷ ν ∷ []) "John.12.3"
∷ word (μ ∷ ύ ∷ ρ ∷ ο ∷ υ ∷ []) "John.12.3"
∷ word (ν ∷ ά ∷ ρ ∷ δ ∷ ο ∷ υ ∷ []) "John.12.3"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ι ∷ κ ∷ ῆ ∷ ς ∷ []) "John.12.3"
∷ word (π ∷ ο ∷ ∙λ ∷ υ ∷ τ ∷ ί ∷ μ ∷ ο ∷ υ ∷ []) "John.12.3"
∷ word (ἤ ∷ ∙λ ∷ ε ∷ ι ∷ ψ ∷ ε ∷ ν ∷ []) "John.12.3"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.12.3"
∷ word (π ∷ ό ∷ δ ∷ α ∷ ς ∷ []) "John.12.3"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.12.3"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ []) "John.12.3"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.12.3"
∷ word (ἐ ∷ ξ ∷ έ ∷ μ ∷ α ∷ ξ ∷ ε ∷ ν ∷ []) "John.12.3"
∷ word (τ ∷ α ∷ ῖ ∷ ς ∷ []) "John.12.3"
∷ word (θ ∷ ρ ∷ ι ∷ ξ ∷ ὶ ∷ ν ∷ []) "John.12.3"
∷ word (α ∷ ὐ ∷ τ ∷ ῆ ∷ ς ∷ []) "John.12.3"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.12.3"
∷ word (π ∷ ό ∷ δ ∷ α ∷ ς ∷ []) "John.12.3"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.12.3"
∷ word (ἡ ∷ []) "John.12.3"
∷ word (δ ∷ ὲ ∷ []) "John.12.3"
∷ word (ο ∷ ἰ ∷ κ ∷ ί ∷ α ∷ []) "John.12.3"
∷ word (ἐ ∷ π ∷ ∙λ ∷ η ∷ ρ ∷ ώ ∷ θ ∷ η ∷ []) "John.12.3"
∷ word (ἐ ∷ κ ∷ []) "John.12.3"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.12.3"
∷ word (ὀ ∷ σ ∷ μ ∷ ῆ ∷ ς ∷ []) "John.12.3"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.12.3"
∷ word (μ ∷ ύ ∷ ρ ∷ ο ∷ υ ∷ []) "John.12.3"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.12.4"
∷ word (δ ∷ ὲ ∷ []) "John.12.4"
∷ word (Ἰ ∷ ο ∷ ύ ∷ δ ∷ α ∷ ς ∷ []) "John.12.4"
∷ word (ὁ ∷ []) "John.12.4"
∷ word (Ἰ ∷ σ ∷ κ ∷ α ∷ ρ ∷ ι ∷ ώ ∷ τ ∷ η ∷ ς ∷ []) "John.12.4"
∷ word (ε ∷ ἷ ∷ ς ∷ []) "John.12.4"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.12.4"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ ῶ ∷ ν ∷ []) "John.12.4"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.12.4"
∷ word (ὁ ∷ []) "John.12.4"
∷ word (μ ∷ έ ∷ ∙λ ∷ ∙λ ∷ ω ∷ ν ∷ []) "John.12.4"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.12.4"
∷ word (π ∷ α ∷ ρ ∷ α ∷ δ ∷ ι ∷ δ ∷ ό ∷ ν ∷ α ∷ ι ∷ []) "John.12.4"
∷ word (Δ ∷ ι ∷ ὰ ∷ []) "John.12.5"
∷ word (τ ∷ ί ∷ []) "John.12.5"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.12.5"
∷ word (τ ∷ ὸ ∷ []) "John.12.5"
∷ word (μ ∷ ύ ∷ ρ ∷ ο ∷ ν ∷ []) "John.12.5"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.12.5"
∷ word (ἐ ∷ π ∷ ρ ∷ ά ∷ θ ∷ η ∷ []) "John.12.5"
∷ word (τ ∷ ρ ∷ ι ∷ α ∷ κ ∷ ο ∷ σ ∷ ί ∷ ω ∷ ν ∷ []) "John.12.5"
∷ word (δ ∷ η ∷ ν ∷ α ∷ ρ ∷ ί ∷ ω ∷ ν ∷ []) "John.12.5"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.12.5"
∷ word (ἐ ∷ δ ∷ ό ∷ θ ∷ η ∷ []) "John.12.5"
∷ word (π ∷ τ ∷ ω ∷ χ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.12.5"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.12.6"
∷ word (δ ∷ ὲ ∷ []) "John.12.6"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.12.6"
∷ word (ο ∷ ὐ ∷ χ ∷ []) "John.12.6"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.12.6"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.12.6"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.12.6"
∷ word (π ∷ τ ∷ ω ∷ χ ∷ ῶ ∷ ν ∷ []) "John.12.6"
∷ word (ἔ ∷ μ ∷ ε ∷ ∙λ ∷ ε ∷ ν ∷ []) "John.12.6"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.12.6"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ []) "John.12.6"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.12.6"
∷ word (κ ∷ ∙λ ∷ έ ∷ π ∷ τ ∷ η ∷ ς ∷ []) "John.12.6"
∷ word (ἦ ∷ ν ∷ []) "John.12.6"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.12.6"
∷ word (τ ∷ ὸ ∷ []) "John.12.6"
∷ word (γ ∷ ∙λ ∷ ω ∷ σ ∷ σ ∷ ό ∷ κ ∷ ο ∷ μ ∷ ο ∷ ν ∷ []) "John.12.6"
∷ word (ἔ ∷ χ ∷ ω ∷ ν ∷ []) "John.12.6"
∷ word (τ ∷ ὰ ∷ []) "John.12.6"
∷ word (β ∷ α ∷ ∙λ ∷ ∙λ ∷ ό ∷ μ ∷ ε ∷ ν ∷ α ∷ []) "John.12.6"
∷ word (ἐ ∷ β ∷ ά ∷ σ ∷ τ ∷ α ∷ ζ ∷ ε ∷ ν ∷ []) "John.12.6"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.12.7"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.12.7"
∷ word (ὁ ∷ []) "John.12.7"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.12.7"
∷ word (Ἄ ∷ φ ∷ ε ∷ ς ∷ []) "John.12.7"
∷ word (α ∷ ὐ ∷ τ ∷ ή ∷ ν ∷ []) "John.12.7"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.12.7"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.12.7"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.12.7"
∷ word (ἡ ∷ μ ∷ έ ∷ ρ ∷ α ∷ ν ∷ []) "John.12.7"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.12.7"
∷ word (ἐ ∷ ν ∷ τ ∷ α ∷ φ ∷ ι ∷ α ∷ σ ∷ μ ∷ ο ∷ ῦ ∷ []) "John.12.7"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.12.7"
∷ word (τ ∷ η ∷ ρ ∷ ή ∷ σ ∷ ῃ ∷ []) "John.12.7"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ []) "John.12.7"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.12.8"
∷ word (π ∷ τ ∷ ω ∷ χ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.12.8"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.12.8"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ ο ∷ τ ∷ ε ∷ []) "John.12.8"
∷ word (ἔ ∷ χ ∷ ε ∷ τ ∷ ε ∷ []) "John.12.8"
∷ word (μ ∷ ε ∷ θ ∷ []) "John.12.8"
∷ word (ἑ ∷ α ∷ υ ∷ τ ∷ ῶ ∷ ν ∷ []) "John.12.8"
∷ word (ἐ ∷ μ ∷ ὲ ∷ []) "John.12.8"
∷ word (δ ∷ ὲ ∷ []) "John.12.8"
∷ word (ο ∷ ὐ ∷ []) "John.12.8"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ ο ∷ τ ∷ ε ∷ []) "John.12.8"
∷ word (ἔ ∷ χ ∷ ε ∷ τ ∷ ε ∷ []) "John.12.8"
∷ word (Ἔ ∷ γ ∷ ν ∷ ω ∷ []) "John.12.9"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.12.9"
∷ word (ὄ ∷ χ ∷ ∙λ ∷ ο ∷ ς ∷ []) "John.12.9"
∷ word (π ∷ ο ∷ ∙λ ∷ ὺ ∷ ς ∷ []) "John.12.9"
∷ word (ἐ ∷ κ ∷ []) "John.12.9"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.12.9"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ί ∷ ω ∷ ν ∷ []) "John.12.9"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.12.9"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ []) "John.12.9"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.12.9"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.12.9"
∷ word (ἦ ∷ ∙λ ∷ θ ∷ ο ∷ ν ∷ []) "John.12.9"
∷ word (ο ∷ ὐ ∷ []) "John.12.9"
∷ word (δ ∷ ι ∷ ὰ ∷ []) "John.12.9"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.12.9"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ν ∷ []) "John.12.9"
∷ word (μ ∷ ό ∷ ν ∷ ο ∷ ν ∷ []) "John.12.9"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ []) "John.12.9"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.12.9"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.12.9"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.12.9"
∷ word (Λ ∷ ά ∷ ζ ∷ α ∷ ρ ∷ ο ∷ ν ∷ []) "John.12.9"
∷ word (ἴ ∷ δ ∷ ω ∷ σ ∷ ι ∷ ν ∷ []) "John.12.9"
∷ word (ὃ ∷ ν ∷ []) "John.12.9"
∷ word (ἤ ∷ γ ∷ ε ∷ ι ∷ ρ ∷ ε ∷ ν ∷ []) "John.12.9"
∷ word (ἐ ∷ κ ∷ []) "John.12.9"
∷ word (ν ∷ ε ∷ κ ∷ ρ ∷ ῶ ∷ ν ∷ []) "John.12.9"
∷ word (ἐ ∷ β ∷ ο ∷ υ ∷ ∙λ ∷ ε ∷ ύ ∷ σ ∷ α ∷ ν ∷ τ ∷ ο ∷ []) "John.12.10"
∷ word (δ ∷ ὲ ∷ []) "John.12.10"
∷ word (ο ∷ ἱ ∷ []) "John.12.10"
∷ word (ἀ ∷ ρ ∷ χ ∷ ι ∷ ε ∷ ρ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.12.10"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.12.10"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.12.10"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.12.10"
∷ word (Λ ∷ ά ∷ ζ ∷ α ∷ ρ ∷ ο ∷ ν ∷ []) "John.12.10"
∷ word (ἀ ∷ π ∷ ο ∷ κ ∷ τ ∷ ε ∷ ί ∷ ν ∷ ω ∷ σ ∷ ι ∷ ν ∷ []) "John.12.10"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.12.11"
∷ word (π ∷ ο ∷ ∙λ ∷ ∙λ ∷ ο ∷ ὶ ∷ []) "John.12.11"
∷ word (δ ∷ ι ∷ []) "John.12.11"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.12.11"
∷ word (ὑ ∷ π ∷ ῆ ∷ γ ∷ ο ∷ ν ∷ []) "John.12.11"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.12.11"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ί ∷ ω ∷ ν ∷ []) "John.12.11"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.12.11"
∷ word (ἐ ∷ π ∷ ί ∷ σ ∷ τ ∷ ε ∷ υ ∷ ο ∷ ν ∷ []) "John.12.11"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.12.11"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.12.11"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ν ∷ []) "John.12.11"
∷ word (Τ ∷ ῇ ∷ []) "John.12.12"
∷ word (ἐ ∷ π ∷ α ∷ ύ ∷ ρ ∷ ι ∷ ο ∷ ν ∷ []) "John.12.12"
∷ word (ὁ ∷ []) "John.12.12"
∷ word (ὄ ∷ χ ∷ ∙λ ∷ ο ∷ ς ∷ []) "John.12.12"
∷ word (π ∷ ο ∷ ∙λ ∷ ὺ ∷ ς ∷ []) "John.12.12"
∷ word (ὁ ∷ []) "John.12.12"
∷ word (ἐ ∷ ∙λ ∷ θ ∷ ὼ ∷ ν ∷ []) "John.12.12"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.12.12"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.12.12"
∷ word (ἑ ∷ ο ∷ ρ ∷ τ ∷ ή ∷ ν ∷ []) "John.12.12"
∷ word (ἀ ∷ κ ∷ ο ∷ ύ ∷ σ ∷ α ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.12.12"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.12.12"
∷ word (ἔ ∷ ρ ∷ χ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.12.12"
∷ word (ὁ ∷ []) "John.12.12"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.12.12"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.12.12"
∷ word (Ἱ ∷ ε ∷ ρ ∷ ο ∷ σ ∷ ό ∷ ∙λ ∷ υ ∷ μ ∷ α ∷ []) "John.12.12"
∷ word (ἔ ∷ ∙λ ∷ α ∷ β ∷ ο ∷ ν ∷ []) "John.12.13"
∷ word (τ ∷ ὰ ∷ []) "John.12.13"
∷ word (β ∷ α ∷ ΐ ∷ α ∷ []) "John.12.13"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.12.13"
∷ word (φ ∷ ο ∷ ι ∷ ν ∷ ί ∷ κ ∷ ω ∷ ν ∷ []) "John.12.13"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.12.13"
∷ word (ἐ ∷ ξ ∷ ῆ ∷ ∙λ ∷ θ ∷ ο ∷ ν ∷ []) "John.12.13"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.12.13"
∷ word (ὑ ∷ π ∷ ά ∷ ν ∷ τ ∷ η ∷ σ ∷ ι ∷ ν ∷ []) "John.12.13"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.12.13"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.12.13"
∷ word (ἐ ∷ κ ∷ ρ ∷ α ∷ ύ ∷ γ ∷ α ∷ ζ ∷ ο ∷ ν ∷ []) "John.12.13"
∷ word (Ὡ ∷ σ ∷ α ∷ ν ∷ ν ∷ ά ∷ []) "John.12.13"
∷ word (ε ∷ ὐ ∷ ∙λ ∷ ο ∷ γ ∷ η ∷ μ ∷ έ ∷ ν ∷ ο ∷ ς ∷ []) "John.12.13"
∷ word (ὁ ∷ []) "John.12.13"
∷ word (ἐ ∷ ρ ∷ χ ∷ ό ∷ μ ∷ ε ∷ ν ∷ ο ∷ ς ∷ []) "John.12.13"
∷ word (ἐ ∷ ν ∷ []) "John.12.13"
∷ word (ὀ ∷ ν ∷ ό ∷ μ ∷ α ∷ τ ∷ ι ∷ []) "John.12.13"
∷ word (κ ∷ υ ∷ ρ ∷ ί ∷ ο ∷ υ ∷ []) "John.12.13"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.12.13"
∷ word (ὁ ∷ []) "John.12.13"
∷ word (β ∷ α ∷ σ ∷ ι ∷ ∙λ ∷ ε ∷ ὺ ∷ ς ∷ []) "John.12.13"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.12.13"
∷ word (Ἰ ∷ σ ∷ ρ ∷ α ∷ ή ∷ ∙λ ∷ []) "John.12.13"
∷ word (ε ∷ ὑ ∷ ρ ∷ ὼ ∷ ν ∷ []) "John.12.14"
∷ word (δ ∷ ὲ ∷ []) "John.12.14"
∷ word (ὁ ∷ []) "John.12.14"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.12.14"
∷ word (ὀ ∷ ν ∷ ά ∷ ρ ∷ ι ∷ ο ∷ ν ∷ []) "John.12.14"
∷ word (ἐ ∷ κ ∷ ά ∷ θ ∷ ι ∷ σ ∷ ε ∷ ν ∷ []) "John.12.14"
∷ word (ἐ ∷ π ∷ []) "John.12.14"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ []) "John.12.14"
∷ word (κ ∷ α ∷ θ ∷ ώ ∷ ς ∷ []) "John.12.14"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.12.14"
∷ word (γ ∷ ε ∷ γ ∷ ρ ∷ α ∷ μ ∷ μ ∷ έ ∷ ν ∷ ο ∷ ν ∷ []) "John.12.14"
∷ word (Μ ∷ ὴ ∷ []) "John.12.15"
∷ word (φ ∷ ο ∷ β ∷ ο ∷ ῦ ∷ []) "John.12.15"
∷ word (θ ∷ υ ∷ γ ∷ ά ∷ τ ∷ η ∷ ρ ∷ []) "John.12.15"
∷ word (Σ ∷ ι ∷ ώ ∷ ν ∷ []) "John.12.15"
∷ word (ἰ ∷ δ ∷ ο ∷ ὺ ∷ []) "John.12.15"
∷ word (ὁ ∷ []) "John.12.15"
∷ word (β ∷ α ∷ σ ∷ ι ∷ ∙λ ∷ ε ∷ ύ ∷ ς ∷ []) "John.12.15"
∷ word (σ ∷ ο ∷ υ ∷ []) "John.12.15"
∷ word (ἔ ∷ ρ ∷ χ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.12.15"
∷ word (κ ∷ α ∷ θ ∷ ή ∷ μ ∷ ε ∷ ν ∷ ο ∷ ς ∷ []) "John.12.15"
∷ word (ἐ ∷ π ∷ ὶ ∷ []) "John.12.15"
∷ word (π ∷ ῶ ∷ ∙λ ∷ ο ∷ ν ∷ []) "John.12.15"
∷ word (ὄ ∷ ν ∷ ο ∷ υ ∷ []) "John.12.15"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.12.16"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.12.16"
∷ word (ἔ ∷ γ ∷ ν ∷ ω ∷ σ ∷ α ∷ ν ∷ []) "John.12.16"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.12.16"
∷ word (ο ∷ ἱ ∷ []) "John.12.16"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ α ∷ ὶ ∷ []) "John.12.16"
∷ word (τ ∷ ὸ ∷ []) "John.12.16"
∷ word (π ∷ ρ ∷ ῶ ∷ τ ∷ ο ∷ ν ∷ []) "John.12.16"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ []) "John.12.16"
∷ word (ὅ ∷ τ ∷ ε ∷ []) "John.12.16"
∷ word (ἐ ∷ δ ∷ ο ∷ ξ ∷ ά ∷ σ ∷ θ ∷ η ∷ []) "John.12.16"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.12.16"
∷ word (τ ∷ ό ∷ τ ∷ ε ∷ []) "John.12.16"
∷ word (ἐ ∷ μ ∷ ν ∷ ή ∷ σ ∷ θ ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.12.16"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.12.16"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.12.16"
∷ word (ἦ ∷ ν ∷ []) "John.12.16"
∷ word (ἐ ∷ π ∷ []) "John.12.16"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.12.16"
∷ word (γ ∷ ε ∷ γ ∷ ρ ∷ α ∷ μ ∷ μ ∷ έ ∷ ν ∷ α ∷ []) "John.12.16"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.12.16"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.12.16"
∷ word (ἐ ∷ π ∷ ο ∷ ί ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.12.16"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.12.16"
∷ word (ἐ ∷ μ ∷ α ∷ ρ ∷ τ ∷ ύ ∷ ρ ∷ ε ∷ ι ∷ []) "John.12.17"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.12.17"
∷ word (ὁ ∷ []) "John.12.17"
∷ word (ὄ ∷ χ ∷ ∙λ ∷ ο ∷ ς ∷ []) "John.12.17"
∷ word (ὁ ∷ []) "John.12.17"
∷ word (ὢ ∷ ν ∷ []) "John.12.17"
∷ word (μ ∷ ε ∷ τ ∷ []) "John.12.17"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.12.17"
∷ word (ὅ ∷ τ ∷ ε ∷ []) "John.12.17"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.12.17"
∷ word (Λ ∷ ά ∷ ζ ∷ α ∷ ρ ∷ ο ∷ ν ∷ []) "John.12.17"
∷ word (ἐ ∷ φ ∷ ώ ∷ ν ∷ η ∷ σ ∷ ε ∷ ν ∷ []) "John.12.17"
∷ word (ἐ ∷ κ ∷ []) "John.12.17"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.12.17"
∷ word (μ ∷ ν ∷ η ∷ μ ∷ ε ∷ ί ∷ ο ∷ υ ∷ []) "John.12.17"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.12.17"
∷ word (ἤ ∷ γ ∷ ε ∷ ι ∷ ρ ∷ ε ∷ ν ∷ []) "John.12.17"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.12.17"
∷ word (ἐ ∷ κ ∷ []) "John.12.17"
∷ word (ν ∷ ε ∷ κ ∷ ρ ∷ ῶ ∷ ν ∷ []) "John.12.17"
∷ word (δ ∷ ι ∷ ὰ ∷ []) "John.12.18"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.12.18"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.12.18"
∷ word (ὑ ∷ π ∷ ή ∷ ν ∷ τ ∷ η ∷ σ ∷ ε ∷ ν ∷ []) "John.12.18"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.12.18"
∷ word (ὁ ∷ []) "John.12.18"
∷ word (ὄ ∷ χ ∷ ∙λ ∷ ο ∷ ς ∷ []) "John.12.18"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.12.18"
∷ word (ἤ ∷ κ ∷ ο ∷ υ ∷ σ ∷ α ∷ ν ∷ []) "John.12.18"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.12.18"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.12.18"
∷ word (π ∷ ε ∷ π ∷ ο ∷ ι ∷ η ∷ κ ∷ έ ∷ ν ∷ α ∷ ι ∷ []) "John.12.18"
∷ word (τ ∷ ὸ ∷ []) "John.12.18"
∷ word (σ ∷ η ∷ μ ∷ ε ∷ ῖ ∷ ο ∷ ν ∷ []) "John.12.18"
∷ word (ο ∷ ἱ ∷ []) "John.12.19"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.12.19"
∷ word (Φ ∷ α ∷ ρ ∷ ι ∷ σ ∷ α ∷ ῖ ∷ ο ∷ ι ∷ []) "John.12.19"
∷ word (ε ∷ ἶ ∷ π ∷ α ∷ ν ∷ []) "John.12.19"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.12.19"
∷ word (ἑ ∷ α ∷ υ ∷ τ ∷ ο ∷ ύ ∷ ς ∷ []) "John.12.19"
∷ word (Θ ∷ ε ∷ ω ∷ ρ ∷ ε ∷ ῖ ∷ τ ∷ ε ∷ []) "John.12.19"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.12.19"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.12.19"
∷ word (ὠ ∷ φ ∷ ε ∷ ∙λ ∷ ε ∷ ῖ ∷ τ ∷ ε ∷ []) "John.12.19"
∷ word (ο ∷ ὐ ∷ δ ∷ έ ∷ ν ∷ []) "John.12.19"
∷ word (ἴ ∷ δ ∷ ε ∷ []) "John.12.19"
∷ word (ὁ ∷ []) "John.12.19"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ ς ∷ []) "John.12.19"
∷ word (ὀ ∷ π ∷ ί ∷ σ ∷ ω ∷ []) "John.12.19"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.12.19"
∷ word (ἀ ∷ π ∷ ῆ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.12.19"
∷ word (Ἦ ∷ σ ∷ α ∷ ν ∷ []) "John.12.20"
∷ word (δ ∷ ὲ ∷ []) "John.12.20"
∷ word (Ἕ ∷ ∙λ ∷ ∙λ ∷ η ∷ ν ∷ έ ∷ ς ∷ []) "John.12.20"
∷ word (τ ∷ ι ∷ ν ∷ ε ∷ ς ∷ []) "John.12.20"
∷ word (ἐ ∷ κ ∷ []) "John.12.20"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.12.20"
∷ word (ἀ ∷ ν ∷ α ∷ β ∷ α ∷ ι ∷ ν ∷ ό ∷ ν ∷ τ ∷ ω ∷ ν ∷ []) "John.12.20"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.12.20"
∷ word (π ∷ ρ ∷ ο ∷ σ ∷ κ ∷ υ ∷ ν ∷ ή ∷ σ ∷ ω ∷ σ ∷ ι ∷ ν ∷ []) "John.12.20"
∷ word (ἐ ∷ ν ∷ []) "John.12.20"
∷ word (τ ∷ ῇ ∷ []) "John.12.20"
∷ word (ἑ ∷ ο ∷ ρ ∷ τ ∷ ῇ ∷ []) "John.12.20"
∷ word (ο ∷ ὗ ∷ τ ∷ ο ∷ ι ∷ []) "John.12.21"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.12.21"
∷ word (π ∷ ρ ∷ ο ∷ σ ∷ ῆ ∷ ∙λ ∷ θ ∷ ο ∷ ν ∷ []) "John.12.21"
∷ word (Φ ∷ ι ∷ ∙λ ∷ ί ∷ π ∷ π ∷ ῳ ∷ []) "John.12.21"
∷ word (τ ∷ ῷ ∷ []) "John.12.21"
∷ word (ἀ ∷ π ∷ ὸ ∷ []) "John.12.21"
∷ word (Β ∷ η ∷ θ ∷ σ ∷ α ∷ ϊ ∷ δ ∷ ὰ ∷ []) "John.12.21"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.12.21"
∷ word (Γ ∷ α ∷ ∙λ ∷ ι ∷ ∙λ ∷ α ∷ ί ∷ α ∷ ς ∷ []) "John.12.21"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.12.21"
∷ word (ἠ ∷ ρ ∷ ώ ∷ τ ∷ ω ∷ ν ∷ []) "John.12.21"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.12.21"
∷ word (∙λ ∷ έ ∷ γ ∷ ο ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.12.21"
∷ word (Κ ∷ ύ ∷ ρ ∷ ι ∷ ε ∷ []) "John.12.21"
∷ word (θ ∷ έ ∷ ∙λ ∷ ο ∷ μ ∷ ε ∷ ν ∷ []) "John.12.21"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.12.21"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ν ∷ []) "John.12.21"
∷ word (ἰ ∷ δ ∷ ε ∷ ῖ ∷ ν ∷ []) "John.12.21"
∷ word (ἔ ∷ ρ ∷ χ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.12.22"
∷ word (ὁ ∷ []) "John.12.22"
∷ word (Φ ∷ ί ∷ ∙λ ∷ ι ∷ π ∷ π ∷ ο ∷ ς ∷ []) "John.12.22"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.12.22"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.12.22"
∷ word (τ ∷ ῷ ∷ []) "John.12.22"
∷ word (Ἀ ∷ ν ∷ δ ∷ ρ ∷ έ ∷ ᾳ ∷ []) "John.12.22"
∷ word (ἔ ∷ ρ ∷ χ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.12.22"
∷ word (Ἀ ∷ ν ∷ δ ∷ ρ ∷ έ ∷ α ∷ ς ∷ []) "John.12.22"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.12.22"
∷ word (Φ ∷ ί ∷ ∙λ ∷ ι ∷ π ∷ π ∷ ο ∷ ς ∷ []) "John.12.22"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.12.22"
∷ word (∙λ ∷ έ ∷ γ ∷ ο ∷ υ ∷ σ ∷ ι ∷ ν ∷ []) "John.12.22"
∷ word (τ ∷ ῷ ∷ []) "John.12.22"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ []) "John.12.22"
∷ word (ὁ ∷ []) "John.12.23"
∷ word (δ ∷ ὲ ∷ []) "John.12.23"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.12.23"
∷ word (ἀ ∷ π ∷ ο ∷ κ ∷ ρ ∷ ί ∷ ν ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.12.23"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.12.23"
∷ word (∙λ ∷ έ ∷ γ ∷ ω ∷ ν ∷ []) "John.12.23"
∷ word (Ἐ ∷ ∙λ ∷ ή ∷ ∙λ ∷ υ ∷ θ ∷ ε ∷ ν ∷ []) "John.12.23"
∷ word (ἡ ∷ []) "John.12.23"
∷ word (ὥ ∷ ρ ∷ α ∷ []) "John.12.23"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.12.23"
∷ word (δ ∷ ο ∷ ξ ∷ α ∷ σ ∷ θ ∷ ῇ ∷ []) "John.12.23"
∷ word (ὁ ∷ []) "John.12.23"
∷ word (υ ∷ ἱ ∷ ὸ ∷ ς ∷ []) "John.12.23"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.12.23"
∷ word (ἀ ∷ ν ∷ θ ∷ ρ ∷ ώ ∷ π ∷ ο ∷ υ ∷ []) "John.12.23"
∷ word (ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.12.24"
∷ word (ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.12.24"
∷ word (∙λ ∷ έ ∷ γ ∷ ω ∷ []) "John.12.24"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.12.24"
∷ word (ἐ ∷ ὰ ∷ ν ∷ []) "John.12.24"
∷ word (μ ∷ ὴ ∷ []) "John.12.24"
∷ word (ὁ ∷ []) "John.12.24"
∷ word (κ ∷ ό ∷ κ ∷ κ ∷ ο ∷ ς ∷ []) "John.12.24"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.12.24"
∷ word (σ ∷ ί ∷ τ ∷ ο ∷ υ ∷ []) "John.12.24"
∷ word (π ∷ ε ∷ σ ∷ ὼ ∷ ν ∷ []) "John.12.24"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.12.24"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.12.24"
∷ word (γ ∷ ῆ ∷ ν ∷ []) "John.12.24"
∷ word (ἀ ∷ π ∷ ο ∷ θ ∷ ά ∷ ν ∷ ῃ ∷ []) "John.12.24"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ς ∷ []) "John.12.24"
∷ word (μ ∷ ό ∷ ν ∷ ο ∷ ς ∷ []) "John.12.24"
∷ word (μ ∷ έ ∷ ν ∷ ε ∷ ι ∷ []) "John.12.24"
∷ word (ἐ ∷ ὰ ∷ ν ∷ []) "John.12.24"
∷ word (δ ∷ ὲ ∷ []) "John.12.24"
∷ word (ἀ ∷ π ∷ ο ∷ θ ∷ ά ∷ ν ∷ ῃ ∷ []) "John.12.24"
∷ word (π ∷ ο ∷ ∙λ ∷ ὺ ∷ ν ∷ []) "John.12.24"
∷ word (κ ∷ α ∷ ρ ∷ π ∷ ὸ ∷ ν ∷ []) "John.12.24"
∷ word (φ ∷ έ ∷ ρ ∷ ε ∷ ι ∷ []) "John.12.24"
∷ word (ὁ ∷ []) "John.12.25"
∷ word (φ ∷ ι ∷ ∙λ ∷ ῶ ∷ ν ∷ []) "John.12.25"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.12.25"
∷ word (ψ ∷ υ ∷ χ ∷ ὴ ∷ ν ∷ []) "John.12.25"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.12.25"
∷ word (ἀ ∷ π ∷ ο ∷ ∙λ ∷ ∙λ ∷ ύ ∷ ε ∷ ι ∷ []) "John.12.25"
∷ word (α ∷ ὐ ∷ τ ∷ ή ∷ ν ∷ []) "John.12.25"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.12.25"
∷ word (ὁ ∷ []) "John.12.25"
∷ word (μ ∷ ι ∷ σ ∷ ῶ ∷ ν ∷ []) "John.12.25"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.12.25"
∷ word (ψ ∷ υ ∷ χ ∷ ὴ ∷ ν ∷ []) "John.12.25"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.12.25"
∷ word (ἐ ∷ ν ∷ []) "John.12.25"
∷ word (τ ∷ ῷ ∷ []) "John.12.25"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ῳ ∷ []) "John.12.25"
∷ word (τ ∷ ο ∷ ύ ∷ τ ∷ ῳ ∷ []) "John.12.25"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.12.25"
∷ word (ζ ∷ ω ∷ ὴ ∷ ν ∷ []) "John.12.25"
∷ word (α ∷ ἰ ∷ ώ ∷ ν ∷ ι ∷ ο ∷ ν ∷ []) "John.12.25"
∷ word (φ ∷ υ ∷ ∙λ ∷ ά ∷ ξ ∷ ε ∷ ι ∷ []) "John.12.25"
∷ word (α ∷ ὐ ∷ τ ∷ ή ∷ ν ∷ []) "John.12.25"
∷ word (ἐ ∷ ὰ ∷ ν ∷ []) "John.12.26"
∷ word (ἐ ∷ μ ∷ ο ∷ ί ∷ []) "John.12.26"
∷ word (τ ∷ ι ∷ ς ∷ []) "John.12.26"
∷ word (δ ∷ ι ∷ α ∷ κ ∷ ο ∷ ν ∷ ῇ ∷ []) "John.12.26"
∷ word (ἐ ∷ μ ∷ ο ∷ ὶ ∷ []) "John.12.26"
∷ word (ἀ ∷ κ ∷ ο ∷ ∙λ ∷ ο ∷ υ ∷ θ ∷ ε ∷ ί ∷ τ ∷ ω ∷ []) "John.12.26"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.12.26"
∷ word (ὅ ∷ π ∷ ο ∷ υ ∷ []) "John.12.26"
∷ word (ε ∷ ἰ ∷ μ ∷ ὶ ∷ []) "John.12.26"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.12.26"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ []) "John.12.26"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.12.26"
∷ word (ὁ ∷ []) "John.12.26"
∷ word (δ ∷ ι ∷ ά ∷ κ ∷ ο ∷ ν ∷ ο ∷ ς ∷ []) "John.12.26"
∷ word (ὁ ∷ []) "John.12.26"
∷ word (ἐ ∷ μ ∷ ὸ ∷ ς ∷ []) "John.12.26"
∷ word (ἔ ∷ σ ∷ τ ∷ α ∷ ι ∷ []) "John.12.26"
∷ word (ἐ ∷ ά ∷ ν ∷ []) "John.12.26"
∷ word (τ ∷ ι ∷ ς ∷ []) "John.12.26"
∷ word (ἐ ∷ μ ∷ ο ∷ ὶ ∷ []) "John.12.26"
∷ word (δ ∷ ι ∷ α ∷ κ ∷ ο ∷ ν ∷ ῇ ∷ []) "John.12.26"
∷ word (τ ∷ ι ∷ μ ∷ ή ∷ σ ∷ ε ∷ ι ∷ []) "John.12.26"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.12.26"
∷ word (ὁ ∷ []) "John.12.26"
∷ word (π ∷ α ∷ τ ∷ ή ∷ ρ ∷ []) "John.12.26"
∷ word (Ν ∷ ῦ ∷ ν ∷ []) "John.12.27"
∷ word (ἡ ∷ []) "John.12.27"
∷ word (ψ ∷ υ ∷ χ ∷ ή ∷ []) "John.12.27"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.12.27"
∷ word (τ ∷ ε ∷ τ ∷ ά ∷ ρ ∷ α ∷ κ ∷ τ ∷ α ∷ ι ∷ []) "John.12.27"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.12.27"
∷ word (τ ∷ ί ∷ []) "John.12.27"
∷ word (ε ∷ ἴ ∷ π ∷ ω ∷ []) "John.12.27"
∷ word (π ∷ ά ∷ τ ∷ ε ∷ ρ ∷ []) "John.12.27"
∷ word (σ ∷ ῶ ∷ σ ∷ ό ∷ ν ∷ []) "John.12.27"
∷ word (μ ∷ ε ∷ []) "John.12.27"
∷ word (ἐ ∷ κ ∷ []) "John.12.27"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.12.27"
∷ word (ὥ ∷ ρ ∷ α ∷ ς ∷ []) "John.12.27"
∷ word (τ ∷ α ∷ ύ ∷ τ ∷ η ∷ ς ∷ []) "John.12.27"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.12.27"
∷ word (δ ∷ ι ∷ ὰ ∷ []) "John.12.27"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.12.27"
∷ word (ἦ ∷ ∙λ ∷ θ ∷ ο ∷ ν ∷ []) "John.12.27"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.12.27"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.12.27"
∷ word (ὥ ∷ ρ ∷ α ∷ ν ∷ []) "John.12.27"
∷ word (τ ∷ α ∷ ύ ∷ τ ∷ η ∷ ν ∷ []) "John.12.27"
∷ word (π ∷ ά ∷ τ ∷ ε ∷ ρ ∷ []) "John.12.28"
∷ word (δ ∷ ό ∷ ξ ∷ α ∷ σ ∷ ό ∷ ν ∷ []) "John.12.28"
∷ word (σ ∷ ο ∷ υ ∷ []) "John.12.28"
∷ word (τ ∷ ὸ ∷ []) "John.12.28"
∷ word (ὄ ∷ ν ∷ ο ∷ μ ∷ α ∷ []) "John.12.28"
∷ word (ἦ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.12.28"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.12.28"
∷ word (φ ∷ ω ∷ ν ∷ ὴ ∷ []) "John.12.28"
∷ word (ἐ ∷ κ ∷ []) "John.12.28"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.12.28"
∷ word (ο ∷ ὐ ∷ ρ ∷ α ∷ ν ∷ ο ∷ ῦ ∷ []) "John.12.28"
∷ word (Κ ∷ α ∷ ὶ ∷ []) "John.12.28"
∷ word (ἐ ∷ δ ∷ ό ∷ ξ ∷ α ∷ σ ∷ α ∷ []) "John.12.28"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.12.28"
∷ word (π ∷ ά ∷ ∙λ ∷ ι ∷ ν ∷ []) "John.12.28"
∷ word (δ ∷ ο ∷ ξ ∷ ά ∷ σ ∷ ω ∷ []) "John.12.28"
∷ word (ὁ ∷ []) "John.12.29"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.12.29"
∷ word (ὄ ∷ χ ∷ ∙λ ∷ ο ∷ ς ∷ []) "John.12.29"
∷ word (ὁ ∷ []) "John.12.29"
∷ word (ἑ ∷ σ ∷ τ ∷ ὼ ∷ ς ∷ []) "John.12.29"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.12.29"
∷ word (ἀ ∷ κ ∷ ο ∷ ύ ∷ σ ∷ α ∷ ς ∷ []) "John.12.29"
∷ word (ἔ ∷ ∙λ ∷ ε ∷ γ ∷ ε ∷ ν ∷ []) "John.12.29"
∷ word (β ∷ ρ ∷ ο ∷ ν ∷ τ ∷ ὴ ∷ ν ∷ []) "John.12.29"
∷ word (γ ∷ ε ∷ γ ∷ ο ∷ ν ∷ έ ∷ ν ∷ α ∷ ι ∷ []) "John.12.29"
∷ word (ἄ ∷ ∙λ ∷ ∙λ ∷ ο ∷ ι ∷ []) "John.12.29"
∷ word (ἔ ∷ ∙λ ∷ ε ∷ γ ∷ ο ∷ ν ∷ []) "John.12.29"
∷ word (Ἄ ∷ γ ∷ γ ∷ ε ∷ ∙λ ∷ ο ∷ ς ∷ []) "John.12.29"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.12.29"
∷ word (∙λ ∷ ε ∷ ∙λ ∷ ά ∷ ∙λ ∷ η ∷ κ ∷ ε ∷ ν ∷ []) "John.12.29"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.12.30"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.12.30"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.12.30"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.12.30"
∷ word (Ο ∷ ὐ ∷ []) "John.12.30"
∷ word (δ ∷ ι ∷ []) "John.12.30"
∷ word (ἐ ∷ μ ∷ ὲ ∷ []) "John.12.30"
∷ word (ἡ ∷ []) "John.12.30"
∷ word (φ ∷ ω ∷ ν ∷ ὴ ∷ []) "John.12.30"
∷ word (α ∷ ὕ ∷ τ ∷ η ∷ []) "John.12.30"
∷ word (γ ∷ έ ∷ γ ∷ ο ∷ ν ∷ ε ∷ ν ∷ []) "John.12.30"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.12.30"
∷ word (δ ∷ ι ∷ []) "John.12.30"
∷ word (ὑ ∷ μ ∷ ᾶ ∷ ς ∷ []) "John.12.30"
∷ word (ν ∷ ῦ ∷ ν ∷ []) "John.12.31"
∷ word (κ ∷ ρ ∷ ί ∷ σ ∷ ι ∷ ς ∷ []) "John.12.31"
∷ word (ἐ ∷ σ ∷ τ ∷ ὶ ∷ ν ∷ []) "John.12.31"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.12.31"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ υ ∷ []) "John.12.31"
∷ word (τ ∷ ο ∷ ύ ∷ τ ∷ ο ∷ υ ∷ []) "John.12.31"
∷ word (ν ∷ ῦ ∷ ν ∷ []) "John.12.31"
∷ word (ὁ ∷ []) "John.12.31"
∷ word (ἄ ∷ ρ ∷ χ ∷ ω ∷ ν ∷ []) "John.12.31"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.12.31"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ υ ∷ []) "John.12.31"
∷ word (τ ∷ ο ∷ ύ ∷ τ ∷ ο ∷ υ ∷ []) "John.12.31"
∷ word (ἐ ∷ κ ∷ β ∷ ∙λ ∷ η ∷ θ ∷ ή ∷ σ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.12.31"
∷ word (ἔ ∷ ξ ∷ ω ∷ []) "John.12.31"
∷ word (κ ∷ ἀ ∷ γ ∷ ὼ ∷ []) "John.12.32"
∷ word (ἐ ∷ ὰ ∷ ν ∷ []) "John.12.32"
∷ word (ὑ ∷ ψ ∷ ω ∷ θ ∷ ῶ ∷ []) "John.12.32"
∷ word (ἐ ∷ κ ∷ []) "John.12.32"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.12.32"
∷ word (γ ∷ ῆ ∷ ς ∷ []) "John.12.32"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ α ∷ ς ∷ []) "John.12.32"
∷ word (ἑ ∷ ∙λ ∷ κ ∷ ύ ∷ σ ∷ ω ∷ []) "John.12.32"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.12.32"
∷ word (ἐ ∷ μ ∷ α ∷ υ ∷ τ ∷ ό ∷ ν ∷ []) "John.12.32"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.12.33"
∷ word (δ ∷ ὲ ∷ []) "John.12.33"
∷ word (ἔ ∷ ∙λ ∷ ε ∷ γ ∷ ε ∷ ν ∷ []) "John.12.33"
∷ word (σ ∷ η ∷ μ ∷ α ∷ ί ∷ ν ∷ ω ∷ ν ∷ []) "John.12.33"
∷ word (π ∷ ο ∷ ί ∷ ῳ ∷ []) "John.12.33"
∷ word (θ ∷ α ∷ ν ∷ ά ∷ τ ∷ ῳ ∷ []) "John.12.33"
∷ word (ἤ ∷ μ ∷ ε ∷ ∙λ ∷ ∙λ ∷ ε ∷ ν ∷ []) "John.12.33"
∷ word (ἀ ∷ π ∷ ο ∷ θ ∷ ν ∷ ῄ ∷ σ ∷ κ ∷ ε ∷ ι ∷ ν ∷ []) "John.12.33"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.12.34"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.12.34"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.12.34"
∷ word (ὁ ∷ []) "John.12.34"
∷ word (ὄ ∷ χ ∷ ∙λ ∷ ο ∷ ς ∷ []) "John.12.34"
∷ word (Ἡ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.12.34"
∷ word (ἠ ∷ κ ∷ ο ∷ ύ ∷ σ ∷ α ∷ μ ∷ ε ∷ ν ∷ []) "John.12.34"
∷ word (ἐ ∷ κ ∷ []) "John.12.34"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.12.34"
∷ word (ν ∷ ό ∷ μ ∷ ο ∷ υ ∷ []) "John.12.34"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.12.34"
∷ word (ὁ ∷ []) "John.12.34"
∷ word (χ ∷ ρ ∷ ι ∷ σ ∷ τ ∷ ὸ ∷ ς ∷ []) "John.12.34"
∷ word (μ ∷ έ ∷ ν ∷ ε ∷ ι ∷ []) "John.12.34"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.12.34"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.12.34"
∷ word (α ∷ ἰ ∷ ῶ ∷ ν ∷ α ∷ []) "John.12.34"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.12.34"
∷ word (π ∷ ῶ ∷ ς ∷ []) "John.12.34"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ ς ∷ []) "John.12.34"
∷ word (σ ∷ ὺ ∷ []) "John.12.34"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.12.34"
∷ word (δ ∷ ε ∷ ῖ ∷ []) "John.12.34"
∷ word (ὑ ∷ ψ ∷ ω ∷ θ ∷ ῆ ∷ ν ∷ α ∷ ι ∷ []) "John.12.34"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.12.34"
∷ word (υ ∷ ἱ ∷ ὸ ∷ ν ∷ []) "John.12.34"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.12.34"
∷ word (ἀ ∷ ν ∷ θ ∷ ρ ∷ ώ ∷ π ∷ ο ∷ υ ∷ []) "John.12.34"
∷ word (τ ∷ ί ∷ ς ∷ []) "John.12.34"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.12.34"
∷ word (ο ∷ ὗ ∷ τ ∷ ο ∷ ς ∷ []) "John.12.34"
∷ word (ὁ ∷ []) "John.12.34"
∷ word (υ ∷ ἱ ∷ ὸ ∷ ς ∷ []) "John.12.34"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.12.34"
∷ word (ἀ ∷ ν ∷ θ ∷ ρ ∷ ώ ∷ π ∷ ο ∷ υ ∷ []) "John.12.34"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.12.35"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.12.35"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.12.35"
∷ word (ὁ ∷ []) "John.12.35"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.12.35"
∷ word (Ἔ ∷ τ ∷ ι ∷ []) "John.12.35"
∷ word (μ ∷ ι ∷ κ ∷ ρ ∷ ὸ ∷ ν ∷ []) "John.12.35"
∷ word (χ ∷ ρ ∷ ό ∷ ν ∷ ο ∷ ν ∷ []) "John.12.35"
∷ word (τ ∷ ὸ ∷ []) "John.12.35"
∷ word (φ ∷ ῶ ∷ ς ∷ []) "John.12.35"
∷ word (ἐ ∷ ν ∷ []) "John.12.35"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.12.35"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.12.35"
∷ word (π ∷ ε ∷ ρ ∷ ι ∷ π ∷ α ∷ τ ∷ ε ∷ ῖ ∷ τ ∷ ε ∷ []) "John.12.35"
∷ word (ὡ ∷ ς ∷ []) "John.12.35"
∷ word (τ ∷ ὸ ∷ []) "John.12.35"
∷ word (φ ∷ ῶ ∷ ς ∷ []) "John.12.35"
∷ word (ἔ ∷ χ ∷ ε ∷ τ ∷ ε ∷ []) "John.12.35"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.12.35"
∷ word (μ ∷ ὴ ∷ []) "John.12.35"
∷ word (σ ∷ κ ∷ ο ∷ τ ∷ ί ∷ α ∷ []) "John.12.35"
∷ word (ὑ ∷ μ ∷ ᾶ ∷ ς ∷ []) "John.12.35"
∷ word (κ ∷ α ∷ τ ∷ α ∷ ∙λ ∷ ά ∷ β ∷ ῃ ∷ []) "John.12.35"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.12.35"
∷ word (ὁ ∷ []) "John.12.35"
∷ word (π ∷ ε ∷ ρ ∷ ι ∷ π ∷ α ∷ τ ∷ ῶ ∷ ν ∷ []) "John.12.35"
∷ word (ἐ ∷ ν ∷ []) "John.12.35"
∷ word (τ ∷ ῇ ∷ []) "John.12.35"
∷ word (σ ∷ κ ∷ ο ∷ τ ∷ ί ∷ ᾳ ∷ []) "John.12.35"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.12.35"
∷ word (ο ∷ ἶ ∷ δ ∷ ε ∷ ν ∷ []) "John.12.35"
∷ word (π ∷ ο ∷ ῦ ∷ []) "John.12.35"
∷ word (ὑ ∷ π ∷ ά ∷ γ ∷ ε ∷ ι ∷ []) "John.12.35"
∷ word (ὡ ∷ ς ∷ []) "John.12.36"
∷ word (τ ∷ ὸ ∷ []) "John.12.36"
∷ word (φ ∷ ῶ ∷ ς ∷ []) "John.12.36"
∷ word (ἔ ∷ χ ∷ ε ∷ τ ∷ ε ∷ []) "John.12.36"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ ε ∷ τ ∷ ε ∷ []) "John.12.36"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.12.36"
∷ word (τ ∷ ὸ ∷ []) "John.12.36"
∷ word (φ ∷ ῶ ∷ ς ∷ []) "John.12.36"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.12.36"
∷ word (υ ∷ ἱ ∷ ο ∷ ὶ ∷ []) "John.12.36"
∷ word (φ ∷ ω ∷ τ ∷ ὸ ∷ ς ∷ []) "John.12.36"
∷ word (γ ∷ έ ∷ ν ∷ η ∷ σ ∷ θ ∷ ε ∷ []) "John.12.36"
∷ word (Τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.12.36"
∷ word (ἐ ∷ ∙λ ∷ ά ∷ ∙λ ∷ η ∷ σ ∷ ε ∷ ν ∷ []) "John.12.36"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.12.36"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.12.36"
∷ word (ἀ ∷ π ∷ ε ∷ ∙λ ∷ θ ∷ ὼ ∷ ν ∷ []) "John.12.36"
∷ word (ἐ ∷ κ ∷ ρ ∷ ύ ∷ β ∷ η ∷ []) "John.12.36"
∷ word (ἀ ∷ π ∷ []) "John.12.36"
∷ word (α ∷ ὐ ∷ τ ∷ ῶ ∷ ν ∷ []) "John.12.36"
∷ word (τ ∷ ο ∷ σ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.12.37"
∷ word (δ ∷ ὲ ∷ []) "John.12.37"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.12.37"
∷ word (σ ∷ η ∷ μ ∷ ε ∷ ῖ ∷ α ∷ []) "John.12.37"
∷ word (π ∷ ε ∷ π ∷ ο ∷ ι ∷ η ∷ κ ∷ ό ∷ τ ∷ ο ∷ ς ∷ []) "John.12.37"
∷ word (ἔ ∷ μ ∷ π ∷ ρ ∷ ο ∷ σ ∷ θ ∷ ε ∷ ν ∷ []) "John.12.37"
∷ word (α ∷ ὐ ∷ τ ∷ ῶ ∷ ν ∷ []) "John.12.37"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.12.37"
∷ word (ἐ ∷ π ∷ ί ∷ σ ∷ τ ∷ ε ∷ υ ∷ ο ∷ ν ∷ []) "John.12.37"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.12.37"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.12.37"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.12.38"
∷ word (ὁ ∷ []) "John.12.38"
∷ word (∙λ ∷ ό ∷ γ ∷ ο ∷ ς ∷ []) "John.12.38"
∷ word (Ἠ ∷ σ ∷ α ∷ ΐ ∷ ο ∷ υ ∷ []) "John.12.38"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.12.38"
∷ word (π ∷ ρ ∷ ο ∷ φ ∷ ή ∷ τ ∷ ο ∷ υ ∷ []) "John.12.38"
∷ word (π ∷ ∙λ ∷ η ∷ ρ ∷ ω ∷ θ ∷ ῇ ∷ []) "John.12.38"
∷ word (ὃ ∷ ν ∷ []) "John.12.38"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.12.38"
∷ word (Κ ∷ ύ ∷ ρ ∷ ι ∷ ε ∷ []) "John.12.38"
∷ word (τ ∷ ί ∷ ς ∷ []) "John.12.38"
∷ word (ἐ ∷ π ∷ ί ∷ σ ∷ τ ∷ ε ∷ υ ∷ σ ∷ ε ∷ ν ∷ []) "John.12.38"
∷ word (τ ∷ ῇ ∷ []) "John.12.38"
∷ word (ἀ ∷ κ ∷ ο ∷ ῇ ∷ []) "John.12.38"
∷ word (ἡ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.12.38"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.12.38"
∷ word (ὁ ∷ []) "John.12.38"
∷ word (β ∷ ρ ∷ α ∷ χ ∷ ί ∷ ω ∷ ν ∷ []) "John.12.38"
∷ word (κ ∷ υ ∷ ρ ∷ ί ∷ ο ∷ υ ∷ []) "John.12.38"
∷ word (τ ∷ ί ∷ ν ∷ ι ∷ []) "John.12.38"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ α ∷ ∙λ ∷ ύ ∷ φ ∷ θ ∷ η ∷ []) "John.12.38"
∷ word (δ ∷ ι ∷ ὰ ∷ []) "John.12.39"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.12.39"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.12.39"
∷ word (ἠ ∷ δ ∷ ύ ∷ ν ∷ α ∷ ν ∷ τ ∷ ο ∷ []) "John.12.39"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ ε ∷ ι ∷ ν ∷ []) "John.12.39"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.12.39"
∷ word (π ∷ ά ∷ ∙λ ∷ ι ∷ ν ∷ []) "John.12.39"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.12.39"
∷ word (Ἠ ∷ σ ∷ α ∷ ΐ ∷ α ∷ ς ∷ []) "John.12.39"
∷ word (Τ ∷ ε ∷ τ ∷ ύ ∷ φ ∷ ∙λ ∷ ω ∷ κ ∷ ε ∷ ν ∷ []) "John.12.40"
∷ word (α ∷ ὐ ∷ τ ∷ ῶ ∷ ν ∷ []) "John.12.40"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.12.40"
∷ word (ὀ ∷ φ ∷ θ ∷ α ∷ ∙λ ∷ μ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.12.40"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.12.40"
∷ word (ἐ ∷ π ∷ ώ ∷ ρ ∷ ω ∷ σ ∷ ε ∷ ν ∷ []) "John.12.40"
∷ word (α ∷ ὐ ∷ τ ∷ ῶ ∷ ν ∷ []) "John.12.40"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.12.40"
∷ word (κ ∷ α ∷ ρ ∷ δ ∷ ί ∷ α ∷ ν ∷ []) "John.12.40"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.12.40"
∷ word (μ ∷ ὴ ∷ []) "John.12.40"
∷ word (ἴ ∷ δ ∷ ω ∷ σ ∷ ι ∷ ν ∷ []) "John.12.40"
∷ word (τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.12.40"
∷ word (ὀ ∷ φ ∷ θ ∷ α ∷ ∙λ ∷ μ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.12.40"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.12.40"
∷ word (ν ∷ ο ∷ ή ∷ σ ∷ ω ∷ σ ∷ ι ∷ ν ∷ []) "John.12.40"
∷ word (τ ∷ ῇ ∷ []) "John.12.40"
∷ word (κ ∷ α ∷ ρ ∷ δ ∷ ί ∷ ᾳ ∷ []) "John.12.40"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.12.40"
∷ word (σ ∷ τ ∷ ρ ∷ α ∷ φ ∷ ῶ ∷ σ ∷ ι ∷ ν ∷ []) "John.12.40"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.12.40"
∷ word (ἰ ∷ ά ∷ σ ∷ ο ∷ μ ∷ α ∷ ι ∷ []) "John.12.40"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ύ ∷ ς ∷ []) "John.12.40"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.12.41"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.12.41"
∷ word (Ἠ ∷ σ ∷ α ∷ ΐ ∷ α ∷ ς ∷ []) "John.12.41"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.12.41"
∷ word (ε ∷ ἶ ∷ δ ∷ ε ∷ ν ∷ []) "John.12.41"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.12.41"
∷ word (δ ∷ ό ∷ ξ ∷ α ∷ ν ∷ []) "John.12.41"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.12.41"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.12.41"
∷ word (ἐ ∷ ∙λ ∷ ά ∷ ∙λ ∷ η ∷ σ ∷ ε ∷ ν ∷ []) "John.12.41"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.12.41"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.12.41"
∷ word (ὅ ∷ μ ∷ ω ∷ ς ∷ []) "John.12.42"
∷ word (μ ∷ έ ∷ ν ∷ τ ∷ ο ∷ ι ∷ []) "John.12.42"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.12.42"
∷ word (ἐ ∷ κ ∷ []) "John.12.42"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.12.42"
∷ word (ἀ ∷ ρ ∷ χ ∷ ό ∷ ν ∷ τ ∷ ω ∷ ν ∷ []) "John.12.42"
∷ word (π ∷ ο ∷ ∙λ ∷ ∙λ ∷ ο ∷ ὶ ∷ []) "John.12.42"
∷ word (ἐ ∷ π ∷ ί ∷ σ ∷ τ ∷ ε ∷ υ ∷ σ ∷ α ∷ ν ∷ []) "John.12.42"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.12.42"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.12.42"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.12.42"
∷ word (δ ∷ ι ∷ ὰ ∷ []) "John.12.42"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.12.42"
∷ word (Φ ∷ α ∷ ρ ∷ ι ∷ σ ∷ α ∷ ί ∷ ο ∷ υ ∷ ς ∷ []) "John.12.42"
∷ word (ο ∷ ὐ ∷ χ ∷ []) "John.12.42"
∷ word (ὡ ∷ μ ∷ ο ∷ ∙λ ∷ ό ∷ γ ∷ ο ∷ υ ∷ ν ∷ []) "John.12.42"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.12.42"
∷ word (μ ∷ ὴ ∷ []) "John.12.42"
∷ word (ἀ ∷ π ∷ ο ∷ σ ∷ υ ∷ ν ∷ ά ∷ γ ∷ ω ∷ γ ∷ ο ∷ ι ∷ []) "John.12.42"
∷ word (γ ∷ έ ∷ ν ∷ ω ∷ ν ∷ τ ∷ α ∷ ι ∷ []) "John.12.42"
∷ word (ἠ ∷ γ ∷ ά ∷ π ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.12.43"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.12.43"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.12.43"
∷ word (δ ∷ ό ∷ ξ ∷ α ∷ ν ∷ []) "John.12.43"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.12.43"
∷ word (ἀ ∷ ν ∷ θ ∷ ρ ∷ ώ ∷ π ∷ ω ∷ ν ∷ []) "John.12.43"
∷ word (μ ∷ ᾶ ∷ ∙λ ∷ ∙λ ∷ ο ∷ ν ∷ []) "John.12.43"
∷ word (ἤ ∷ π ∷ ε ∷ ρ ∷ []) "John.12.43"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.12.43"
∷ word (δ ∷ ό ∷ ξ ∷ α ∷ ν ∷ []) "John.12.43"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.12.43"
∷ word (θ ∷ ε ∷ ο ∷ ῦ ∷ []) "John.12.43"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.12.44"
∷ word (δ ∷ ὲ ∷ []) "John.12.44"
∷ word (ἔ ∷ κ ∷ ρ ∷ α ∷ ξ ∷ ε ∷ ν ∷ []) "John.12.44"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.12.44"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.12.44"
∷ word (Ὁ ∷ []) "John.12.44"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ ω ∷ ν ∷ []) "John.12.44"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.12.44"
∷ word (ἐ ∷ μ ∷ ὲ ∷ []) "John.12.44"
∷ word (ο ∷ ὐ ∷ []) "John.12.44"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ ε ∷ ι ∷ []) "John.12.44"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.12.44"
∷ word (ἐ ∷ μ ∷ ὲ ∷ []) "John.12.44"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.12.44"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.12.44"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.12.44"
∷ word (π ∷ έ ∷ μ ∷ ψ ∷ α ∷ ν ∷ τ ∷ ά ∷ []) "John.12.44"
∷ word (μ ∷ ε ∷ []) "John.12.44"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.12.45"
∷ word (ὁ ∷ []) "John.12.45"
∷ word (θ ∷ ε ∷ ω ∷ ρ ∷ ῶ ∷ ν ∷ []) "John.12.45"
∷ word (ἐ ∷ μ ∷ ὲ ∷ []) "John.12.45"
∷ word (θ ∷ ε ∷ ω ∷ ρ ∷ ε ∷ ῖ ∷ []) "John.12.45"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.12.45"
∷ word (π ∷ έ ∷ μ ∷ ψ ∷ α ∷ ν ∷ τ ∷ ά ∷ []) "John.12.45"
∷ word (μ ∷ ε ∷ []) "John.12.45"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.12.46"
∷ word (φ ∷ ῶ ∷ ς ∷ []) "John.12.46"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.12.46"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.12.46"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ ν ∷ []) "John.12.46"
∷ word (ἐ ∷ ∙λ ∷ ή ∷ ∙λ ∷ υ ∷ θ ∷ α ∷ []) "John.12.46"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.12.46"
∷ word (π ∷ ᾶ ∷ ς ∷ []) "John.12.46"
∷ word (ὁ ∷ []) "John.12.46"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ ω ∷ ν ∷ []) "John.12.46"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.12.46"
∷ word (ἐ ∷ μ ∷ ὲ ∷ []) "John.12.46"
∷ word (ἐ ∷ ν ∷ []) "John.12.46"
∷ word (τ ∷ ῇ ∷ []) "John.12.46"
∷ word (σ ∷ κ ∷ ο ∷ τ ∷ ί ∷ ᾳ ∷ []) "John.12.46"
∷ word (μ ∷ ὴ ∷ []) "John.12.46"
∷ word (μ ∷ ε ∷ ί ∷ ν ∷ ῃ ∷ []) "John.12.46"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.12.47"
∷ word (ἐ ∷ ά ∷ ν ∷ []) "John.12.47"
∷ word (τ ∷ ί ∷ ς ∷ []) "John.12.47"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.12.47"
∷ word (ἀ ∷ κ ∷ ο ∷ ύ ∷ σ ∷ ῃ ∷ []) "John.12.47"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.12.47"
∷ word (ῥ ∷ η ∷ μ ∷ ά ∷ τ ∷ ω ∷ ν ∷ []) "John.12.47"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.12.47"
∷ word (μ ∷ ὴ ∷ []) "John.12.47"
∷ word (φ ∷ υ ∷ ∙λ ∷ ά ∷ ξ ∷ ῃ ∷ []) "John.12.47"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.12.47"
∷ word (ο ∷ ὐ ∷ []) "John.12.47"
∷ word (κ ∷ ρ ∷ ί ∷ ν ∷ ω ∷ []) "John.12.47"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.12.47"
∷ word (ο ∷ ὐ ∷ []) "John.12.47"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.12.47"
∷ word (ἦ ∷ ∙λ ∷ θ ∷ ο ∷ ν ∷ []) "John.12.47"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.12.47"
∷ word (κ ∷ ρ ∷ ί ∷ ν ∷ ω ∷ []) "John.12.47"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.12.47"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ ν ∷ []) "John.12.47"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ []) "John.12.47"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.12.47"
∷ word (σ ∷ ώ ∷ σ ∷ ω ∷ []) "John.12.47"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.12.47"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ ν ∷ []) "John.12.47"
∷ word (ὁ ∷ []) "John.12.48"
∷ word (ἀ ∷ θ ∷ ε ∷ τ ∷ ῶ ∷ ν ∷ []) "John.12.48"
∷ word (ἐ ∷ μ ∷ ὲ ∷ []) "John.12.48"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.12.48"
∷ word (μ ∷ ὴ ∷ []) "John.12.48"
∷ word (∙λ ∷ α ∷ μ ∷ β ∷ ά ∷ ν ∷ ω ∷ ν ∷ []) "John.12.48"
∷ word (τ ∷ ὰ ∷ []) "John.12.48"
∷ word (ῥ ∷ ή ∷ μ ∷ α ∷ τ ∷ ά ∷ []) "John.12.48"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.12.48"
∷ word (ἔ ∷ χ ∷ ε ∷ ι ∷ []) "John.12.48"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.12.48"
∷ word (κ ∷ ρ ∷ ί ∷ ν ∷ ο ∷ ν ∷ τ ∷ α ∷ []) "John.12.48"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.12.48"
∷ word (ὁ ∷ []) "John.12.48"
∷ word (∙λ ∷ ό ∷ γ ∷ ο ∷ ς ∷ []) "John.12.48"
∷ word (ὃ ∷ ν ∷ []) "John.12.48"
∷ word (ἐ ∷ ∙λ ∷ ά ∷ ∙λ ∷ η ∷ σ ∷ α ∷ []) "John.12.48"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ο ∷ ς ∷ []) "John.12.48"
∷ word (κ ∷ ρ ∷ ι ∷ ν ∷ ε ∷ ῖ ∷ []) "John.12.48"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.12.48"
∷ word (ἐ ∷ ν ∷ []) "John.12.48"
∷ word (τ ∷ ῇ ∷ []) "John.12.48"
∷ word (ἐ ∷ σ ∷ χ ∷ ά ∷ τ ∷ ῃ ∷ []) "John.12.48"
∷ word (ἡ ∷ μ ∷ έ ∷ ρ ∷ ᾳ ∷ []) "John.12.48"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.12.49"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.12.49"
∷ word (ἐ ∷ ξ ∷ []) "John.12.49"
∷ word (ἐ ∷ μ ∷ α ∷ υ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.12.49"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.12.49"
∷ word (ἐ ∷ ∙λ ∷ ά ∷ ∙λ ∷ η ∷ σ ∷ α ∷ []) "John.12.49"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ []) "John.12.49"
∷ word (ὁ ∷ []) "John.12.49"
∷ word (π ∷ έ ∷ μ ∷ ψ ∷ α ∷ ς ∷ []) "John.12.49"
∷ word (μ ∷ ε ∷ []) "John.12.49"
∷ word (π ∷ α ∷ τ ∷ ὴ ∷ ρ ∷ []) "John.12.49"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ς ∷ []) "John.12.49"
∷ word (μ ∷ ο ∷ ι ∷ []) "John.12.49"
∷ word (ἐ ∷ ν ∷ τ ∷ ο ∷ ∙λ ∷ ὴ ∷ ν ∷ []) "John.12.49"
∷ word (δ ∷ έ ∷ δ ∷ ω ∷ κ ∷ ε ∷ ν ∷ []) "John.12.49"
∷ word (τ ∷ ί ∷ []) "John.12.49"
∷ word (ε ∷ ἴ ∷ π ∷ ω ∷ []) "John.12.49"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.12.49"
∷ word (τ ∷ ί ∷ []) "John.12.49"
∷ word (∙λ ∷ α ∷ ∙λ ∷ ή ∷ σ ∷ ω ∷ []) "John.12.49"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.12.50"
∷ word (ο ∷ ἶ ∷ δ ∷ α ∷ []) "John.12.50"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.12.50"
∷ word (ἡ ∷ []) "John.12.50"
∷ word (ἐ ∷ ν ∷ τ ∷ ο ∷ ∙λ ∷ ὴ ∷ []) "John.12.50"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.12.50"
∷ word (ζ ∷ ω ∷ ὴ ∷ []) "John.12.50"
∷ word (α ∷ ἰ ∷ ώ ∷ ν ∷ ι ∷ ό ∷ ς ∷ []) "John.12.50"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.12.50"
∷ word (ἃ ∷ []) "John.12.50"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.12.50"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.12.50"
∷ word (∙λ ∷ α ∷ ∙λ ∷ ῶ ∷ []) "John.12.50"
∷ word (κ ∷ α ∷ θ ∷ ὼ ∷ ς ∷ []) "John.12.50"
∷ word (ε ∷ ἴ ∷ ρ ∷ η ∷ κ ∷ έ ∷ ν ∷ []) "John.12.50"
∷ word (μ ∷ ο ∷ ι ∷ []) "John.12.50"
∷ word (ὁ ∷ []) "John.12.50"
∷ word (π ∷ α ∷ τ ∷ ή ∷ ρ ∷ []) "John.12.50"
∷ word (ο ∷ ὕ ∷ τ ∷ ω ∷ ς ∷ []) "John.12.50"
∷ word (∙λ ∷ α ∷ ∙λ ∷ ῶ ∷ []) "John.12.50"
∷ word (Π ∷ ρ ∷ ὸ ∷ []) "John.13.1"
∷ word (δ ∷ ὲ ∷ []) "John.13.1"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.13.1"
∷ word (ἑ ∷ ο ∷ ρ ∷ τ ∷ ῆ ∷ ς ∷ []) "John.13.1"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.13.1"
∷ word (π ∷ ά ∷ σ ∷ χ ∷ α ∷ []) "John.13.1"
∷ word (ε ∷ ἰ ∷ δ ∷ ὼ ∷ ς ∷ []) "John.13.1"
∷ word (ὁ ∷ []) "John.13.1"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.13.1"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.13.1"
∷ word (ἦ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.13.1"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.13.1"
∷ word (ἡ ∷ []) "John.13.1"
∷ word (ὥ ∷ ρ ∷ α ∷ []) "John.13.1"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.13.1"
∷ word (μ ∷ ε ∷ τ ∷ α ∷ β ∷ ῇ ∷ []) "John.13.1"
∷ word (ἐ ∷ κ ∷ []) "John.13.1"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.13.1"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ υ ∷ []) "John.13.1"
∷ word (τ ∷ ο ∷ ύ ∷ τ ∷ ο ∷ υ ∷ []) "John.13.1"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.13.1"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.13.1"
∷ word (π ∷ α ∷ τ ∷ έ ∷ ρ ∷ α ∷ []) "John.13.1"
∷ word (ἀ ∷ γ ∷ α ∷ π ∷ ή ∷ σ ∷ α ∷ ς ∷ []) "John.13.1"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.13.1"
∷ word (ἰ ∷ δ ∷ ί ∷ ο ∷ υ ∷ ς ∷ []) "John.13.1"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.13.1"
∷ word (ἐ ∷ ν ∷ []) "John.13.1"
∷ word (τ ∷ ῷ ∷ []) "John.13.1"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ῳ ∷ []) "John.13.1"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.13.1"
∷ word (τ ∷ έ ∷ ∙λ ∷ ο ∷ ς ∷ []) "John.13.1"
∷ word (ἠ ∷ γ ∷ ά ∷ π ∷ η ∷ σ ∷ ε ∷ ν ∷ []) "John.13.1"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ύ ∷ ς ∷ []) "John.13.1"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.13.2"
∷ word (δ ∷ ε ∷ ί ∷ π ∷ ν ∷ ο ∷ υ ∷ []) "John.13.2"
∷ word (γ ∷ ι ∷ ν ∷ ο ∷ μ ∷ έ ∷ ν ∷ ο ∷ υ ∷ []) "John.13.2"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.13.2"
∷ word (δ ∷ ι ∷ α ∷ β ∷ ό ∷ ∙λ ∷ ο ∷ υ ∷ []) "John.13.2"
∷ word (ἤ ∷ δ ∷ η ∷ []) "John.13.2"
∷ word (β ∷ ε ∷ β ∷ ∙λ ∷ η ∷ κ ∷ ό ∷ τ ∷ ο ∷ ς ∷ []) "John.13.2"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.13.2"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.13.2"
∷ word (κ ∷ α ∷ ρ ∷ δ ∷ ί ∷ α ∷ ν ∷ []) "John.13.2"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.13.2"
∷ word (π ∷ α ∷ ρ ∷ α ∷ δ ∷ ο ∷ ῖ ∷ []) "John.13.2"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.13.2"
∷ word (Ἰ ∷ ο ∷ ύ ∷ δ ∷ α ∷ ς ∷ []) "John.13.2"
∷ word (Σ ∷ ί ∷ μ ∷ ω ∷ ν ∷ ο ∷ ς ∷ []) "John.13.2"
∷ word (Ἰ ∷ σ ∷ κ ∷ α ∷ ρ ∷ ι ∷ ώ ∷ τ ∷ ο ∷ υ ∷ []) "John.13.2"
∷ word (ε ∷ ἰ ∷ δ ∷ ὼ ∷ ς ∷ []) "John.13.3"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.13.3"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ α ∷ []) "John.13.3"
∷ word (ἔ ∷ δ ∷ ω ∷ κ ∷ ε ∷ ν ∷ []) "John.13.3"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.13.3"
∷ word (ὁ ∷ []) "John.13.3"
∷ word (π ∷ α ∷ τ ∷ ὴ ∷ ρ ∷ []) "John.13.3"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.13.3"
∷ word (τ ∷ ὰ ∷ ς ∷ []) "John.13.3"
∷ word (χ ∷ ε ∷ ῖ ∷ ρ ∷ α ∷ ς ∷ []) "John.13.3"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.13.3"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.13.3"
∷ word (ἀ ∷ π ∷ ὸ ∷ []) "John.13.3"
∷ word (θ ∷ ε ∷ ο ∷ ῦ ∷ []) "John.13.3"
∷ word (ἐ ∷ ξ ∷ ῆ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.13.3"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.13.3"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.13.3"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.13.3"
∷ word (θ ∷ ε ∷ ὸ ∷ ν ∷ []) "John.13.3"
∷ word (ὑ ∷ π ∷ ά ∷ γ ∷ ε ∷ ι ∷ []) "John.13.3"
∷ word (ἐ ∷ γ ∷ ε ∷ ί ∷ ρ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.13.4"
∷ word (ἐ ∷ κ ∷ []) "John.13.4"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.13.4"
∷ word (δ ∷ ε ∷ ί ∷ π ∷ ν ∷ ο ∷ υ ∷ []) "John.13.4"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.13.4"
∷ word (τ ∷ ί ∷ θ ∷ η ∷ σ ∷ ι ∷ ν ∷ []) "John.13.4"
∷ word (τ ∷ ὰ ∷ []) "John.13.4"
∷ word (ἱ ∷ μ ∷ ά ∷ τ ∷ ι ∷ α ∷ []) "John.13.4"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.13.4"
∷ word (∙λ ∷ α ∷ β ∷ ὼ ∷ ν ∷ []) "John.13.4"
∷ word (∙λ ∷ έ ∷ ν ∷ τ ∷ ι ∷ ο ∷ ν ∷ []) "John.13.4"
∷ word (δ ∷ ι ∷ έ ∷ ζ ∷ ω ∷ σ ∷ ε ∷ ν ∷ []) "John.13.4"
∷ word (ἑ ∷ α ∷ υ ∷ τ ∷ ό ∷ ν ∷ []) "John.13.4"
∷ word (ε ∷ ἶ ∷ τ ∷ α ∷ []) "John.13.5"
∷ word (β ∷ ά ∷ ∙λ ∷ ∙λ ∷ ε ∷ ι ∷ []) "John.13.5"
∷ word (ὕ ∷ δ ∷ ω ∷ ρ ∷ []) "John.13.5"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.13.5"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.13.5"
∷ word (ν ∷ ι ∷ π ∷ τ ∷ ῆ ∷ ρ ∷ α ∷ []) "John.13.5"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.13.5"
∷ word (ἤ ∷ ρ ∷ ξ ∷ α ∷ τ ∷ ο ∷ []) "John.13.5"
∷ word (ν ∷ ί ∷ π ∷ τ ∷ ε ∷ ι ∷ ν ∷ []) "John.13.5"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.13.5"
∷ word (π ∷ ό ∷ δ ∷ α ∷ ς ∷ []) "John.13.5"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.13.5"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ ῶ ∷ ν ∷ []) "John.13.5"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.13.5"
∷ word (ἐ ∷ κ ∷ μ ∷ ά ∷ σ ∷ σ ∷ ε ∷ ι ∷ ν ∷ []) "John.13.5"
∷ word (τ ∷ ῷ ∷ []) "John.13.5"
∷ word (∙λ ∷ ε ∷ ν ∷ τ ∷ ί ∷ ῳ ∷ []) "John.13.5"
∷ word (ᾧ ∷ []) "John.13.5"
∷ word (ἦ ∷ ν ∷ []) "John.13.5"
∷ word (δ ∷ ι ∷ ε ∷ ζ ∷ ω ∷ σ ∷ μ ∷ έ ∷ ν ∷ ο ∷ ς ∷ []) "John.13.5"
∷ word (ἔ ∷ ρ ∷ χ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.13.6"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.13.6"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.13.6"
∷ word (Σ ∷ ί ∷ μ ∷ ω ∷ ν ∷ α ∷ []) "John.13.6"
∷ word (Π ∷ έ ∷ τ ∷ ρ ∷ ο ∷ ν ∷ []) "John.13.6"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.13.6"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.13.6"
∷ word (Κ ∷ ύ ∷ ρ ∷ ι ∷ ε ∷ []) "John.13.6"
∷ word (σ ∷ ύ ∷ []) "John.13.6"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.13.6"
∷ word (ν ∷ ί ∷ π ∷ τ ∷ ε ∷ ι ∷ ς ∷ []) "John.13.6"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.13.6"
∷ word (π ∷ ό ∷ δ ∷ α ∷ ς ∷ []) "John.13.6"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.13.7"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.13.7"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.13.7"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.13.7"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.13.7"
∷ word (Ὃ ∷ []) "John.13.7"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.13.7"
∷ word (π ∷ ο ∷ ι ∷ ῶ ∷ []) "John.13.7"
∷ word (σ ∷ ὺ ∷ []) "John.13.7"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.13.7"
∷ word (ο ∷ ἶ ∷ δ ∷ α ∷ ς ∷ []) "John.13.7"
∷ word (ἄ ∷ ρ ∷ τ ∷ ι ∷ []) "John.13.7"
∷ word (γ ∷ ν ∷ ώ ∷ σ ∷ ῃ ∷ []) "John.13.7"
∷ word (δ ∷ ὲ ∷ []) "John.13.7"
∷ word (μ ∷ ε ∷ τ ∷ ὰ ∷ []) "John.13.7"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.13.7"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.13.8"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.13.8"
∷ word (Π ∷ έ ∷ τ ∷ ρ ∷ ο ∷ ς ∷ []) "John.13.8"
∷ word (Ο ∷ ὐ ∷ []) "John.13.8"
∷ word (μ ∷ ὴ ∷ []) "John.13.8"
∷ word (ν ∷ ί ∷ ψ ∷ ῃ ∷ ς ∷ []) "John.13.8"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.13.8"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.13.8"
∷ word (π ∷ ό ∷ δ ∷ α ∷ ς ∷ []) "John.13.8"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.13.8"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.13.8"
∷ word (α ∷ ἰ ∷ ῶ ∷ ν ∷ α ∷ []) "John.13.8"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.13.8"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.13.8"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.13.8"
∷ word (Ἐ ∷ ὰ ∷ ν ∷ []) "John.13.8"
∷ word (μ ∷ ὴ ∷ []) "John.13.8"
∷ word (ν ∷ ί ∷ ψ ∷ ω ∷ []) "John.13.8"
∷ word (σ ∷ ε ∷ []) "John.13.8"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.13.8"
∷ word (ἔ ∷ χ ∷ ε ∷ ι ∷ ς ∷ []) "John.13.8"
∷ word (μ ∷ έ ∷ ρ ∷ ο ∷ ς ∷ []) "John.13.8"
∷ word (μ ∷ ε ∷ τ ∷ []) "John.13.8"
∷ word (ἐ ∷ μ ∷ ο ∷ ῦ ∷ []) "John.13.8"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.13.9"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.13.9"
∷ word (Σ ∷ ί ∷ μ ∷ ω ∷ ν ∷ []) "John.13.9"
∷ word (Π ∷ έ ∷ τ ∷ ρ ∷ ο ∷ ς ∷ []) "John.13.9"
∷ word (Κ ∷ ύ ∷ ρ ∷ ι ∷ ε ∷ []) "John.13.9"
∷ word (μ ∷ ὴ ∷ []) "John.13.9"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.13.9"
∷ word (π ∷ ό ∷ δ ∷ α ∷ ς ∷ []) "John.13.9"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.13.9"
∷ word (μ ∷ ό ∷ ν ∷ ο ∷ ν ∷ []) "John.13.9"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.13.9"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.13.9"
∷ word (τ ∷ ὰ ∷ ς ∷ []) "John.13.9"
∷ word (χ ∷ ε ∷ ῖ ∷ ρ ∷ α ∷ ς ∷ []) "John.13.9"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.13.9"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.13.9"
∷ word (κ ∷ ε ∷ φ ∷ α ∷ ∙λ ∷ ή ∷ ν ∷ []) "John.13.9"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.13.10"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.13.10"
∷ word (ὁ ∷ []) "John.13.10"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.13.10"
∷ word (Ὁ ∷ []) "John.13.10"
∷ word (∙λ ∷ ε ∷ ∙λ ∷ ο ∷ υ ∷ μ ∷ έ ∷ ν ∷ ο ∷ ς ∷ []) "John.13.10"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.13.10"
∷ word (ἔ ∷ χ ∷ ε ∷ ι ∷ []) "John.13.10"
∷ word (χ ∷ ρ ∷ ε ∷ ί ∷ α ∷ ν ∷ []) "John.13.10"
∷ word (ε ∷ ἰ ∷ []) "John.13.10"
∷ word (μ ∷ ὴ ∷ []) "John.13.10"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.13.10"
∷ word (π ∷ ό ∷ δ ∷ α ∷ ς ∷ []) "John.13.10"
∷ word (ν ∷ ί ∷ ψ ∷ α ∷ σ ∷ θ ∷ α ∷ ι ∷ []) "John.13.10"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ []) "John.13.10"
∷ word (ἔ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.13.10"
∷ word (κ ∷ α ∷ θ ∷ α ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.13.10"
∷ word (ὅ ∷ ∙λ ∷ ο ∷ ς ∷ []) "John.13.10"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.13.10"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.13.10"
∷ word (κ ∷ α ∷ θ ∷ α ∷ ρ ∷ ο ∷ ί ∷ []) "John.13.10"
∷ word (ἐ ∷ σ ∷ τ ∷ ε ∷ []) "John.13.10"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ []) "John.13.10"
∷ word (ο ∷ ὐ ∷ χ ∷ ὶ ∷ []) "John.13.10"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.13.10"
∷ word (ᾔ ∷ δ ∷ ε ∷ ι ∷ []) "John.13.11"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.13.11"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.13.11"
∷ word (π ∷ α ∷ ρ ∷ α ∷ δ ∷ ι ∷ δ ∷ ό ∷ ν ∷ τ ∷ α ∷ []) "John.13.11"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.13.11"
∷ word (δ ∷ ι ∷ ὰ ∷ []) "John.13.11"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.13.11"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.13.11"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.13.11"
∷ word (Ο ∷ ὐ ∷ χ ∷ ὶ ∷ []) "John.13.11"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.13.11"
∷ word (κ ∷ α ∷ θ ∷ α ∷ ρ ∷ ο ∷ ί ∷ []) "John.13.11"
∷ word (ἐ ∷ σ ∷ τ ∷ ε ∷ []) "John.13.11"
∷ word (Ὅ ∷ τ ∷ ε ∷ []) "John.13.12"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.13.12"
∷ word (ἔ ∷ ν ∷ ι ∷ ψ ∷ ε ∷ ν ∷ []) "John.13.12"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.13.12"
∷ word (π ∷ ό ∷ δ ∷ α ∷ ς ∷ []) "John.13.12"
∷ word (α ∷ ὐ ∷ τ ∷ ῶ ∷ ν ∷ []) "John.13.12"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.13.12"
∷ word (ἔ ∷ ∙λ ∷ α ∷ β ∷ ε ∷ ν ∷ []) "John.13.12"
∷ word (τ ∷ ὰ ∷ []) "John.13.12"
∷ word (ἱ ∷ μ ∷ ά ∷ τ ∷ ι ∷ α ∷ []) "John.13.12"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.13.12"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.13.12"
∷ word (ἀ ∷ ν ∷ έ ∷ π ∷ ε ∷ σ ∷ ε ∷ ν ∷ []) "John.13.12"
∷ word (π ∷ ά ∷ ∙λ ∷ ι ∷ ν ∷ []) "John.13.12"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.13.12"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.13.12"
∷ word (Γ ∷ ι ∷ ν ∷ ώ ∷ σ ∷ κ ∷ ε ∷ τ ∷ ε ∷ []) "John.13.12"
∷ word (τ ∷ ί ∷ []) "John.13.12"
∷ word (π ∷ ε ∷ π ∷ ο ∷ ί ∷ η ∷ κ ∷ α ∷ []) "John.13.12"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.13.12"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.13.13"
∷ word (φ ∷ ω ∷ ν ∷ ε ∷ ῖ ∷ τ ∷ έ ∷ []) "John.13.13"
∷ word (μ ∷ ε ∷ []) "John.13.13"
∷ word (Ὁ ∷ []) "John.13.13"
∷ word (δ ∷ ι ∷ δ ∷ ά ∷ σ ∷ κ ∷ α ∷ ∙λ ∷ ο ∷ ς ∷ []) "John.13.13"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.13.13"
∷ word (Ὁ ∷ []) "John.13.13"
∷ word (κ ∷ ύ ∷ ρ ∷ ι ∷ ο ∷ ς ∷ []) "John.13.13"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.13.13"
∷ word (κ ∷ α ∷ ∙λ ∷ ῶ ∷ ς ∷ []) "John.13.13"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ τ ∷ ε ∷ []) "John.13.13"
∷ word (ε ∷ ἰ ∷ μ ∷ ὶ ∷ []) "John.13.13"
∷ word (γ ∷ ά ∷ ρ ∷ []) "John.13.13"
∷ word (ε ∷ ἰ ∷ []) "John.13.14"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.13.14"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.13.14"
∷ word (ἔ ∷ ν ∷ ι ∷ ψ ∷ α ∷ []) "John.13.14"
∷ word (ὑ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.13.14"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.13.14"
∷ word (π ∷ ό ∷ δ ∷ α ∷ ς ∷ []) "John.13.14"
∷ word (ὁ ∷ []) "John.13.14"
∷ word (κ ∷ ύ ∷ ρ ∷ ι ∷ ο ∷ ς ∷ []) "John.13.14"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.13.14"
∷ word (ὁ ∷ []) "John.13.14"
∷ word (δ ∷ ι ∷ δ ∷ ά ∷ σ ∷ κ ∷ α ∷ ∙λ ∷ ο ∷ ς ∷ []) "John.13.14"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.13.14"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.13.14"
∷ word (ὀ ∷ φ ∷ ε ∷ ί ∷ ∙λ ∷ ε ∷ τ ∷ ε ∷ []) "John.13.14"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ή ∷ ∙λ ∷ ω ∷ ν ∷ []) "John.13.14"
∷ word (ν ∷ ί ∷ π ∷ τ ∷ ε ∷ ι ∷ ν ∷ []) "John.13.14"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.13.14"
∷ word (π ∷ ό ∷ δ ∷ α ∷ ς ∷ []) "John.13.14"
∷ word (ὑ ∷ π ∷ ό ∷ δ ∷ ε ∷ ι ∷ γ ∷ μ ∷ α ∷ []) "John.13.15"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.13.15"
∷ word (ἔ ∷ δ ∷ ω ∷ κ ∷ α ∷ []) "John.13.15"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.13.15"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.13.15"
∷ word (κ ∷ α ∷ θ ∷ ὼ ∷ ς ∷ []) "John.13.15"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.13.15"
∷ word (ἐ ∷ π ∷ ο ∷ ί ∷ η ∷ σ ∷ α ∷ []) "John.13.15"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.13.15"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.13.15"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.13.15"
∷ word (π ∷ ο ∷ ι ∷ ῆ ∷ τ ∷ ε ∷ []) "John.13.15"
∷ word (ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.13.16"
∷ word (ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.13.16"
∷ word (∙λ ∷ έ ∷ γ ∷ ω ∷ []) "John.13.16"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.13.16"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.13.16"
∷ word (ἔ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.13.16"
∷ word (δ ∷ ο ∷ ῦ ∷ ∙λ ∷ ο ∷ ς ∷ []) "John.13.16"
∷ word (μ ∷ ε ∷ ί ∷ ζ ∷ ω ∷ ν ∷ []) "John.13.16"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.13.16"
∷ word (κ ∷ υ ∷ ρ ∷ ί ∷ ο ∷ υ ∷ []) "John.13.16"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.13.16"
∷ word (ο ∷ ὐ ∷ δ ∷ ὲ ∷ []) "John.13.16"
∷ word (ἀ ∷ π ∷ ό ∷ σ ∷ τ ∷ ο ∷ ∙λ ∷ ο ∷ ς ∷ []) "John.13.16"
∷ word (μ ∷ ε ∷ ί ∷ ζ ∷ ω ∷ ν ∷ []) "John.13.16"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.13.16"
∷ word (π ∷ έ ∷ μ ∷ ψ ∷ α ∷ ν ∷ τ ∷ ο ∷ ς ∷ []) "John.13.16"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.13.16"
∷ word (ε ∷ ἰ ∷ []) "John.13.17"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.13.17"
∷ word (ο ∷ ἴ ∷ δ ∷ α ∷ τ ∷ ε ∷ []) "John.13.17"
∷ word (μ ∷ α ∷ κ ∷ ά ∷ ρ ∷ ι ∷ ο ∷ ί ∷ []) "John.13.17"
∷ word (ἐ ∷ σ ∷ τ ∷ ε ∷ []) "John.13.17"
∷ word (ἐ ∷ ὰ ∷ ν ∷ []) "John.13.17"
∷ word (π ∷ ο ∷ ι ∷ ῆ ∷ τ ∷ ε ∷ []) "John.13.17"
∷ word (α ∷ ὐ ∷ τ ∷ ά ∷ []) "John.13.17"
∷ word (ο ∷ ὐ ∷ []) "John.13.18"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.13.18"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ ω ∷ ν ∷ []) "John.13.18"
∷ word (ὑ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.13.18"
∷ word (∙λ ∷ έ ∷ γ ∷ ω ∷ []) "John.13.18"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.13.18"
∷ word (ο ∷ ἶ ∷ δ ∷ α ∷ []) "John.13.18"
∷ word (τ ∷ ί ∷ ν ∷ α ∷ ς ∷ []) "John.13.18"
∷ word (ἐ ∷ ξ ∷ ε ∷ ∙λ ∷ ε ∷ ξ ∷ ά ∷ μ ∷ η ∷ ν ∷ []) "John.13.18"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ []) "John.13.18"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.13.18"
∷ word (ἡ ∷ []) "John.13.18"
∷ word (γ ∷ ρ ∷ α ∷ φ ∷ ὴ ∷ []) "John.13.18"
∷ word (π ∷ ∙λ ∷ η ∷ ρ ∷ ω ∷ θ ∷ ῇ ∷ []) "John.13.18"
∷ word (Ὁ ∷ []) "John.13.18"
∷ word (τ ∷ ρ ∷ ώ ∷ γ ∷ ω ∷ ν ∷ []) "John.13.18"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.13.18"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.13.18"
∷ word (ἄ ∷ ρ ∷ τ ∷ ο ∷ ν ∷ []) "John.13.18"
∷ word (ἐ ∷ π ∷ ῆ ∷ ρ ∷ ε ∷ ν ∷ []) "John.13.18"
∷ word (ἐ ∷ π ∷ []) "John.13.18"
∷ word (ἐ ∷ μ ∷ ὲ ∷ []) "John.13.18"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.13.18"
∷ word (π ∷ τ ∷ έ ∷ ρ ∷ ν ∷ α ∷ ν ∷ []) "John.13.18"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.13.18"
∷ word (ἀ ∷ π ∷ []) "John.13.19"
∷ word (ἄ ∷ ρ ∷ τ ∷ ι ∷ []) "John.13.19"
∷ word (∙λ ∷ έ ∷ γ ∷ ω ∷ []) "John.13.19"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.13.19"
∷ word (π ∷ ρ ∷ ὸ ∷ []) "John.13.19"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.13.19"
∷ word (γ ∷ ε ∷ ν ∷ έ ∷ σ ∷ θ ∷ α ∷ ι ∷ []) "John.13.19"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.13.19"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ σ ∷ η ∷ τ ∷ ε ∷ []) "John.13.19"
∷ word (ὅ ∷ τ ∷ α ∷ ν ∷ []) "John.13.19"
∷ word (γ ∷ έ ∷ ν ∷ η ∷ τ ∷ α ∷ ι ∷ []) "John.13.19"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.13.19"
∷ word (ἐ ∷ γ ∷ ώ ∷ []) "John.13.19"
∷ word (ε ∷ ἰ ∷ μ ∷ ι ∷ []) "John.13.19"
∷ word (ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.13.20"
∷ word (ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.13.20"
∷ word (∙λ ∷ έ ∷ γ ∷ ω ∷ []) "John.13.20"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.13.20"
∷ word (ὁ ∷ []) "John.13.20"
∷ word (∙λ ∷ α ∷ μ ∷ β ∷ ά ∷ ν ∷ ω ∷ ν ∷ []) "John.13.20"
∷ word (ἄ ∷ ν ∷ []) "John.13.20"
∷ word (τ ∷ ι ∷ ν ∷ α ∷ []) "John.13.20"
∷ word (π ∷ έ ∷ μ ∷ ψ ∷ ω ∷ []) "John.13.20"
∷ word (ἐ ∷ μ ∷ ὲ ∷ []) "John.13.20"
∷ word (∙λ ∷ α ∷ μ ∷ β ∷ ά ∷ ν ∷ ε ∷ ι ∷ []) "John.13.20"
∷ word (ὁ ∷ []) "John.13.20"
∷ word (δ ∷ ὲ ∷ []) "John.13.20"
∷ word (ἐ ∷ μ ∷ ὲ ∷ []) "John.13.20"
∷ word (∙λ ∷ α ∷ μ ∷ β ∷ ά ∷ ν ∷ ω ∷ ν ∷ []) "John.13.20"
∷ word (∙λ ∷ α ∷ μ ∷ β ∷ ά ∷ ν ∷ ε ∷ ι ∷ []) "John.13.20"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.13.20"
∷ word (π ∷ έ ∷ μ ∷ ψ ∷ α ∷ ν ∷ τ ∷ ά ∷ []) "John.13.20"
∷ word (μ ∷ ε ∷ []) "John.13.20"
∷ word (Τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.13.21"
∷ word (ε ∷ ἰ ∷ π ∷ ὼ ∷ ν ∷ []) "John.13.21"
∷ word (ὁ ∷ []) "John.13.21"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.13.21"
∷ word (ἐ ∷ τ ∷ α ∷ ρ ∷ ά ∷ χ ∷ θ ∷ η ∷ []) "John.13.21"
∷ word (τ ∷ ῷ ∷ []) "John.13.21"
∷ word (π ∷ ν ∷ ε ∷ ύ ∷ μ ∷ α ∷ τ ∷ ι ∷ []) "John.13.21"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.13.21"
∷ word (ἐ ∷ μ ∷ α ∷ ρ ∷ τ ∷ ύ ∷ ρ ∷ η ∷ σ ∷ ε ∷ ν ∷ []) "John.13.21"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.13.21"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.13.21"
∷ word (Ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.13.21"
∷ word (ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.13.21"
∷ word (∙λ ∷ έ ∷ γ ∷ ω ∷ []) "John.13.21"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.13.21"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.13.21"
∷ word (ε ∷ ἷ ∷ ς ∷ []) "John.13.21"
∷ word (ἐ ∷ ξ ∷ []) "John.13.21"
∷ word (ὑ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.13.21"
∷ word (π ∷ α ∷ ρ ∷ α ∷ δ ∷ ώ ∷ σ ∷ ε ∷ ι ∷ []) "John.13.21"
∷ word (μ ∷ ε ∷ []) "John.13.21"
∷ word (ἔ ∷ β ∷ ∙λ ∷ ε ∷ π ∷ ο ∷ ν ∷ []) "John.13.22"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.13.22"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ή ∷ ∙λ ∷ ο ∷ υ ∷ ς ∷ []) "John.13.22"
∷ word (ο ∷ ἱ ∷ []) "John.13.22"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ α ∷ ὶ ∷ []) "John.13.22"
∷ word (ἀ ∷ π ∷ ο ∷ ρ ∷ ο ∷ ύ ∷ μ ∷ ε ∷ ν ∷ ο ∷ ι ∷ []) "John.13.22"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.13.22"
∷ word (τ ∷ ί ∷ ν ∷ ο ∷ ς ∷ []) "John.13.22"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.13.22"
∷ word (ἦ ∷ ν ∷ []) "John.13.23"
∷ word (ἀ ∷ ν ∷ α ∷ κ ∷ ε ∷ ί ∷ μ ∷ ε ∷ ν ∷ ο ∷ ς ∷ []) "John.13.23"
∷ word (ε ∷ ἷ ∷ ς ∷ []) "John.13.23"
∷ word (ἐ ∷ κ ∷ []) "John.13.23"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.13.23"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ ῶ ∷ ν ∷ []) "John.13.23"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.13.23"
∷ word (ἐ ∷ ν ∷ []) "John.13.23"
∷ word (τ ∷ ῷ ∷ []) "John.13.23"
∷ word (κ ∷ ό ∷ ∙λ ∷ π ∷ ῳ ∷ []) "John.13.23"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.13.23"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ []) "John.13.23"
∷ word (ὃ ∷ ν ∷ []) "John.13.23"
∷ word (ἠ ∷ γ ∷ ά ∷ π ∷ α ∷ []) "John.13.23"
∷ word (ὁ ∷ []) "John.13.23"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.13.23"
∷ word (ν ∷ ε ∷ ύ ∷ ε ∷ ι ∷ []) "John.13.24"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.13.24"
∷ word (τ ∷ ο ∷ ύ ∷ τ ∷ ῳ ∷ []) "John.13.24"
∷ word (Σ ∷ ί ∷ μ ∷ ω ∷ ν ∷ []) "John.13.24"
∷ word (Π ∷ έ ∷ τ ∷ ρ ∷ ο ∷ ς ∷ []) "John.13.24"
∷ word (π ∷ υ ∷ θ ∷ έ ∷ σ ∷ θ ∷ α ∷ ι ∷ []) "John.13.24"
∷ word (τ ∷ ί ∷ ς ∷ []) "John.13.24"
∷ word (ἂ ∷ ν ∷ []) "John.13.24"
∷ word (ε ∷ ἴ ∷ η ∷ []) "John.13.24"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.13.24"
∷ word (ο ∷ ὗ ∷ []) "John.13.24"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.13.24"
∷ word (ἀ ∷ ν ∷ α ∷ π ∷ ε ∷ σ ∷ ὼ ∷ ν ∷ []) "John.13.25"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ο ∷ ς ∷ []) "John.13.25"
∷ word (ο ∷ ὕ ∷ τ ∷ ω ∷ ς ∷ []) "John.13.25"
∷ word (ἐ ∷ π ∷ ὶ ∷ []) "John.13.25"
∷ word (τ ∷ ὸ ∷ []) "John.13.25"
∷ word (σ ∷ τ ∷ ῆ ∷ θ ∷ ο ∷ ς ∷ []) "John.13.25"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.13.25"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ []) "John.13.25"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.13.25"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.13.25"
∷ word (Κ ∷ ύ ∷ ρ ∷ ι ∷ ε ∷ []) "John.13.25"
∷ word (τ ∷ ί ∷ ς ∷ []) "John.13.25"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.13.25"
∷ word (ἀ ∷ π ∷ ο ∷ κ ∷ ρ ∷ ί ∷ ν ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.13.26"
∷ word (ὁ ∷ []) "John.13.26"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.13.26"
∷ word (Ἐ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ό ∷ ς ∷ []) "John.13.26"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.13.26"
∷ word (ᾧ ∷ []) "John.13.26"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.13.26"
∷ word (β ∷ ά ∷ ψ ∷ ω ∷ []) "John.13.26"
∷ word (τ ∷ ὸ ∷ []) "John.13.26"
∷ word (ψ ∷ ω ∷ μ ∷ ί ∷ ο ∷ ν ∷ []) "John.13.26"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.13.26"
∷ word (δ ∷ ώ ∷ σ ∷ ω ∷ []) "John.13.26"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.13.26"
∷ word (β ∷ ά ∷ ψ ∷ α ∷ ς ∷ []) "John.13.26"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.13.26"
∷ word (τ ∷ ὸ ∷ []) "John.13.26"
∷ word (ψ ∷ ω ∷ μ ∷ ί ∷ ο ∷ ν ∷ []) "John.13.26"
∷ word (δ ∷ ί ∷ δ ∷ ω ∷ σ ∷ ι ∷ ν ∷ []) "John.13.26"
∷ word (Ἰ ∷ ο ∷ ύ ∷ δ ∷ ᾳ ∷ []) "John.13.26"
∷ word (Σ ∷ ί ∷ μ ∷ ω ∷ ν ∷ ο ∷ ς ∷ []) "John.13.26"
∷ word (Ἰ ∷ σ ∷ κ ∷ α ∷ ρ ∷ ι ∷ ώ ∷ τ ∷ ο ∷ υ ∷ []) "John.13.26"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.13.27"
∷ word (μ ∷ ε ∷ τ ∷ ὰ ∷ []) "John.13.27"
∷ word (τ ∷ ὸ ∷ []) "John.13.27"
∷ word (ψ ∷ ω ∷ μ ∷ ί ∷ ο ∷ ν ∷ []) "John.13.27"
∷ word (τ ∷ ό ∷ τ ∷ ε ∷ []) "John.13.27"
∷ word (ε ∷ ἰ ∷ σ ∷ ῆ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.13.27"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.13.27"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ο ∷ ν ∷ []) "John.13.27"
∷ word (ὁ ∷ []) "John.13.27"
∷ word (Σ ∷ α ∷ τ ∷ α ∷ ν ∷ ᾶ ∷ ς ∷ []) "John.13.27"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.13.27"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.13.27"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.13.27"
∷ word (ὁ ∷ []) "John.13.27"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.13.27"
∷ word (Ὃ ∷ []) "John.13.27"
∷ word (π ∷ ο ∷ ι ∷ ε ∷ ῖ ∷ ς ∷ []) "John.13.27"
∷ word (π ∷ ο ∷ ί ∷ η ∷ σ ∷ ο ∷ ν ∷ []) "John.13.27"
∷ word (τ ∷ ά ∷ χ ∷ ι ∷ ο ∷ ν ∷ []) "John.13.27"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.13.28"
∷ word (δ ∷ ὲ ∷ []) "John.13.28"
∷ word (ο ∷ ὐ ∷ δ ∷ ε ∷ ὶ ∷ ς ∷ []) "John.13.28"
∷ word (ἔ ∷ γ ∷ ν ∷ ω ∷ []) "John.13.28"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.13.28"
∷ word (ἀ ∷ ν ∷ α ∷ κ ∷ ε ∷ ι ∷ μ ∷ έ ∷ ν ∷ ω ∷ ν ∷ []) "John.13.28"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.13.28"
∷ word (τ ∷ ί ∷ []) "John.13.28"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.13.28"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.13.28"
∷ word (τ ∷ ι ∷ ν ∷ ὲ ∷ ς ∷ []) "John.13.29"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.13.29"
∷ word (ἐ ∷ δ ∷ ό ∷ κ ∷ ο ∷ υ ∷ ν ∷ []) "John.13.29"
∷ word (ἐ ∷ π ∷ ε ∷ ὶ ∷ []) "John.13.29"
∷ word (τ ∷ ὸ ∷ []) "John.13.29"
∷ word (γ ∷ ∙λ ∷ ω ∷ σ ∷ σ ∷ ό ∷ κ ∷ ο ∷ μ ∷ ο ∷ ν ∷ []) "John.13.29"
∷ word (ε ∷ ἶ ∷ χ ∷ ε ∷ ν ∷ []) "John.13.29"
∷ word (Ἰ ∷ ο ∷ ύ ∷ δ ∷ α ∷ ς ∷ []) "John.13.29"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.13.29"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.13.29"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.13.29"
∷ word (ὁ ∷ []) "John.13.29"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.13.29"
∷ word (Ἀ ∷ γ ∷ ό ∷ ρ ∷ α ∷ σ ∷ ο ∷ ν ∷ []) "John.13.29"
∷ word (ὧ ∷ ν ∷ []) "John.13.29"
∷ word (χ ∷ ρ ∷ ε ∷ ί ∷ α ∷ ν ∷ []) "John.13.29"
∷ word (ἔ ∷ χ ∷ ο ∷ μ ∷ ε ∷ ν ∷ []) "John.13.29"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.13.29"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.13.29"
∷ word (ἑ ∷ ο ∷ ρ ∷ τ ∷ ή ∷ ν ∷ []) "John.13.29"
∷ word (ἢ ∷ []) "John.13.29"
∷ word (τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.13.29"
∷ word (π ∷ τ ∷ ω ∷ χ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.13.29"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.13.29"
∷ word (τ ∷ ι ∷ []) "John.13.29"
∷ word (δ ∷ ῷ ∷ []) "John.13.29"
∷ word (∙λ ∷ α ∷ β ∷ ὼ ∷ ν ∷ []) "John.13.30"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.13.30"
∷ word (τ ∷ ὸ ∷ []) "John.13.30"
∷ word (ψ ∷ ω ∷ μ ∷ ί ∷ ο ∷ ν ∷ []) "John.13.30"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ο ∷ ς ∷ []) "John.13.30"
∷ word (ἐ ∷ ξ ∷ ῆ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.13.30"
∷ word (ε ∷ ὐ ∷ θ ∷ ύ ∷ ς ∷ []) "John.13.30"
∷ word (ἦ ∷ ν ∷ []) "John.13.30"
∷ word (δ ∷ ὲ ∷ []) "John.13.30"
∷ word (ν ∷ ύ ∷ ξ ∷ []) "John.13.30"
∷ word (Ὅ ∷ τ ∷ ε ∷ []) "John.13.31"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.13.31"
∷ word (ἐ ∷ ξ ∷ ῆ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.13.31"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.13.31"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.13.31"
∷ word (Ν ∷ ῦ ∷ ν ∷ []) "John.13.31"
∷ word (ἐ ∷ δ ∷ ο ∷ ξ ∷ ά ∷ σ ∷ θ ∷ η ∷ []) "John.13.31"
∷ word (ὁ ∷ []) "John.13.31"
∷ word (υ ∷ ἱ ∷ ὸ ∷ ς ∷ []) "John.13.31"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.13.31"
∷ word (ἀ ∷ ν ∷ θ ∷ ρ ∷ ώ ∷ π ∷ ο ∷ υ ∷ []) "John.13.31"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.13.31"
∷ word (ὁ ∷ []) "John.13.31"
∷ word (θ ∷ ε ∷ ὸ ∷ ς ∷ []) "John.13.31"
∷ word (ἐ ∷ δ ∷ ο ∷ ξ ∷ ά ∷ σ ∷ θ ∷ η ∷ []) "John.13.31"
∷ word (ἐ ∷ ν ∷ []) "John.13.31"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.13.31"
∷ word (ε ∷ ἰ ∷ []) "John.13.32"
∷ word (ὁ ∷ []) "John.13.32"
∷ word (θ ∷ ε ∷ ὸ ∷ ς ∷ []) "John.13.32"
∷ word (ἐ ∷ δ ∷ ο ∷ ξ ∷ ά ∷ σ ∷ θ ∷ η ∷ []) "John.13.32"
∷ word (ἐ ∷ ν ∷ []) "John.13.32"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.13.32"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.13.32"
∷ word (ὁ ∷ []) "John.13.32"
∷ word (θ ∷ ε ∷ ὸ ∷ ς ∷ []) "John.13.32"
∷ word (δ ∷ ο ∷ ξ ∷ ά ∷ σ ∷ ε ∷ ι ∷ []) "John.13.32"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.13.32"
∷ word (ἐ ∷ ν ∷ []) "John.13.32"
∷ word (α ∷ ὑ ∷ τ ∷ ῷ ∷ []) "John.13.32"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.13.32"
∷ word (ε ∷ ὐ ∷ θ ∷ ὺ ∷ ς ∷ []) "John.13.32"
∷ word (δ ∷ ο ∷ ξ ∷ ά ∷ σ ∷ ε ∷ ι ∷ []) "John.13.32"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.13.32"
∷ word (τ ∷ ε ∷ κ ∷ ν ∷ ί ∷ α ∷ []) "John.13.33"
∷ word (ἔ ∷ τ ∷ ι ∷ []) "John.13.33"
∷ word (μ ∷ ι ∷ κ ∷ ρ ∷ ὸ ∷ ν ∷ []) "John.13.33"
∷ word (μ ∷ ε ∷ θ ∷ []) "John.13.33"
∷ word (ὑ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.13.33"
∷ word (ε ∷ ἰ ∷ μ ∷ ι ∷ []) "John.13.33"
∷ word (ζ ∷ η ∷ τ ∷ ή ∷ σ ∷ ε ∷ τ ∷ έ ∷ []) "John.13.33"
∷ word (μ ∷ ε ∷ []) "John.13.33"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.13.33"
∷ word (κ ∷ α ∷ θ ∷ ὼ ∷ ς ∷ []) "John.13.33"
∷ word (ε ∷ ἶ ∷ π ∷ ο ∷ ν ∷ []) "John.13.33"
∷ word (τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.13.33"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ί ∷ ο ∷ ι ∷ ς ∷ []) "John.13.33"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.13.33"
∷ word (Ὅ ∷ π ∷ ο ∷ υ ∷ []) "John.13.33"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.13.33"
∷ word (ὑ ∷ π ∷ ά ∷ γ ∷ ω ∷ []) "John.13.33"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.13.33"
∷ word (ο ∷ ὐ ∷ []) "John.13.33"
∷ word (δ ∷ ύ ∷ ν ∷ α ∷ σ ∷ θ ∷ ε ∷ []) "John.13.33"
∷ word (ἐ ∷ ∙λ ∷ θ ∷ ε ∷ ῖ ∷ ν ∷ []) "John.13.33"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.13.33"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.13.33"
∷ word (∙λ ∷ έ ∷ γ ∷ ω ∷ []) "John.13.33"
∷ word (ἄ ∷ ρ ∷ τ ∷ ι ∷ []) "John.13.33"
∷ word (ἐ ∷ ν ∷ τ ∷ ο ∷ ∙λ ∷ ὴ ∷ ν ∷ []) "John.13.34"
∷ word (κ ∷ α ∷ ι ∷ ν ∷ ὴ ∷ ν ∷ []) "John.13.34"
∷ word (δ ∷ ί ∷ δ ∷ ω ∷ μ ∷ ι ∷ []) "John.13.34"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.13.34"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.13.34"
∷ word (ἀ ∷ γ ∷ α ∷ π ∷ ᾶ ∷ τ ∷ ε ∷ []) "John.13.34"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ή ∷ ∙λ ∷ ο ∷ υ ∷ ς ∷ []) "John.13.34"
∷ word (κ ∷ α ∷ θ ∷ ὼ ∷ ς ∷ []) "John.13.34"
∷ word (ἠ ∷ γ ∷ ά ∷ π ∷ η ∷ σ ∷ α ∷ []) "John.13.34"
∷ word (ὑ ∷ μ ∷ ᾶ ∷ ς ∷ []) "John.13.34"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.13.34"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.13.34"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.13.34"
∷ word (ἀ ∷ γ ∷ α ∷ π ∷ ᾶ ∷ τ ∷ ε ∷ []) "John.13.34"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ή ∷ ∙λ ∷ ο ∷ υ ∷ ς ∷ []) "John.13.34"
∷ word (ἐ ∷ ν ∷ []) "John.13.35"
∷ word (τ ∷ ο ∷ ύ ∷ τ ∷ ῳ ∷ []) "John.13.35"
∷ word (γ ∷ ν ∷ ώ ∷ σ ∷ ο ∷ ν ∷ τ ∷ α ∷ ι ∷ []) "John.13.35"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.13.35"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.13.35"
∷ word (ἐ ∷ μ ∷ ο ∷ ὶ ∷ []) "John.13.35"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ α ∷ ί ∷ []) "John.13.35"
∷ word (ἐ ∷ σ ∷ τ ∷ ε ∷ []) "John.13.35"
∷ word (ἐ ∷ ὰ ∷ ν ∷ []) "John.13.35"
∷ word (ἀ ∷ γ ∷ ά ∷ π ∷ η ∷ ν ∷ []) "John.13.35"
∷ word (ἔ ∷ χ ∷ η ∷ τ ∷ ε ∷ []) "John.13.35"
∷ word (ἐ ∷ ν ∷ []) "John.13.35"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ή ∷ ∙λ ∷ ο ∷ ι ∷ ς ∷ []) "John.13.35"
∷ word (Λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.13.36"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.13.36"
∷ word (Σ ∷ ί ∷ μ ∷ ω ∷ ν ∷ []) "John.13.36"
∷ word (Π ∷ έ ∷ τ ∷ ρ ∷ ο ∷ ς ∷ []) "John.13.36"
∷ word (Κ ∷ ύ ∷ ρ ∷ ι ∷ ε ∷ []) "John.13.36"
∷ word (π ∷ ο ∷ ῦ ∷ []) "John.13.36"
∷ word (ὑ ∷ π ∷ ά ∷ γ ∷ ε ∷ ι ∷ ς ∷ []) "John.13.36"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.13.36"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.13.36"
∷ word (Ὅ ∷ π ∷ ο ∷ υ ∷ []) "John.13.36"
∷ word (ὑ ∷ π ∷ ά ∷ γ ∷ ω ∷ []) "John.13.36"
∷ word (ο ∷ ὐ ∷ []) "John.13.36"
∷ word (δ ∷ ύ ∷ ν ∷ α ∷ σ ∷ α ∷ ί ∷ []) "John.13.36"
∷ word (μ ∷ ο ∷ ι ∷ []) "John.13.36"
∷ word (ν ∷ ῦ ∷ ν ∷ []) "John.13.36"
∷ word (ἀ ∷ κ ∷ ο ∷ ∙λ ∷ ο ∷ υ ∷ θ ∷ ῆ ∷ σ ∷ α ∷ ι ∷ []) "John.13.36"
∷ word (ἀ ∷ κ ∷ ο ∷ ∙λ ∷ ο ∷ υ ∷ θ ∷ ή ∷ σ ∷ ε ∷ ι ∷ ς ∷ []) "John.13.36"
∷ word (δ ∷ ὲ ∷ []) "John.13.36"
∷ word (ὕ ∷ σ ∷ τ ∷ ε ∷ ρ ∷ ο ∷ ν ∷ []) "John.13.36"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.13.37"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.13.37"
∷ word (ὁ ∷ []) "John.13.37"
∷ word (Π ∷ έ ∷ τ ∷ ρ ∷ ο ∷ ς ∷ []) "John.13.37"
∷ word (Κ ∷ ύ ∷ ρ ∷ ι ∷ ε ∷ []) "John.13.37"
∷ word (δ ∷ ι ∷ ὰ ∷ []) "John.13.37"
∷ word (τ ∷ ί ∷ []) "John.13.37"
∷ word (ο ∷ ὐ ∷ []) "John.13.37"
∷ word (δ ∷ ύ ∷ ν ∷ α ∷ μ ∷ α ∷ ί ∷ []) "John.13.37"
∷ word (σ ∷ ο ∷ ι ∷ []) "John.13.37"
∷ word (ἀ ∷ κ ∷ ο ∷ ∙λ ∷ ο ∷ υ ∷ θ ∷ ῆ ∷ σ ∷ α ∷ ι ∷ []) "John.13.37"
∷ word (ἄ ∷ ρ ∷ τ ∷ ι ∷ []) "John.13.37"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.13.37"
∷ word (ψ ∷ υ ∷ χ ∷ ή ∷ ν ∷ []) "John.13.37"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.13.37"
∷ word (ὑ ∷ π ∷ ὲ ∷ ρ ∷ []) "John.13.37"
∷ word (σ ∷ ο ∷ ῦ ∷ []) "John.13.37"
∷ word (θ ∷ ή ∷ σ ∷ ω ∷ []) "John.13.37"
∷ word (ἀ ∷ π ∷ ο ∷ κ ∷ ρ ∷ ί ∷ ν ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.13.38"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.13.38"
∷ word (Τ ∷ ὴ ∷ ν ∷ []) "John.13.38"
∷ word (ψ ∷ υ ∷ χ ∷ ή ∷ ν ∷ []) "John.13.38"
∷ word (σ ∷ ο ∷ υ ∷ []) "John.13.38"
∷ word (ὑ ∷ π ∷ ὲ ∷ ρ ∷ []) "John.13.38"
∷ word (ἐ ∷ μ ∷ ο ∷ ῦ ∷ []) "John.13.38"
∷ word (θ ∷ ή ∷ σ ∷ ε ∷ ι ∷ ς ∷ []) "John.13.38"
∷ word (ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.13.38"
∷ word (ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.13.38"
∷ word (∙λ ∷ έ ∷ γ ∷ ω ∷ []) "John.13.38"
∷ word (σ ∷ ο ∷ ι ∷ []) "John.13.38"
∷ word (ο ∷ ὐ ∷ []) "John.13.38"
∷ word (μ ∷ ὴ ∷ []) "John.13.38"
∷ word (ἀ ∷ ∙λ ∷ έ ∷ κ ∷ τ ∷ ω ∷ ρ ∷ []) "John.13.38"
∷ word (φ ∷ ω ∷ ν ∷ ή ∷ σ ∷ ῃ ∷ []) "John.13.38"
∷ word (ἕ ∷ ω ∷ ς ∷ []) "John.13.38"
∷ word (ο ∷ ὗ ∷ []) "John.13.38"
∷ word (ἀ ∷ ρ ∷ ν ∷ ή ∷ σ ∷ ῃ ∷ []) "John.13.38"
∷ word (μ ∷ ε ∷ []) "John.13.38"
∷ word (τ ∷ ρ ∷ ί ∷ ς ∷ []) "John.13.38"
∷ word (Μ ∷ ὴ ∷ []) "John.14.1"
∷ word (τ ∷ α ∷ ρ ∷ α ∷ σ ∷ σ ∷ έ ∷ σ ∷ θ ∷ ω ∷ []) "John.14.1"
∷ word (ὑ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.14.1"
∷ word (ἡ ∷ []) "John.14.1"
∷ word (κ ∷ α ∷ ρ ∷ δ ∷ ί ∷ α ∷ []) "John.14.1"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ ε ∷ τ ∷ ε ∷ []) "John.14.1"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.14.1"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.14.1"
∷ word (θ ∷ ε ∷ ό ∷ ν ∷ []) "John.14.1"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.14.1"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.14.1"
∷ word (ἐ ∷ μ ∷ ὲ ∷ []) "John.14.1"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ ε ∷ τ ∷ ε ∷ []) "John.14.1"
∷ word (ἐ ∷ ν ∷ []) "John.14.2"
∷ word (τ ∷ ῇ ∷ []) "John.14.2"
∷ word (ο ∷ ἰ ∷ κ ∷ ί ∷ ᾳ ∷ []) "John.14.2"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.14.2"
∷ word (π ∷ α ∷ τ ∷ ρ ∷ ό ∷ ς ∷ []) "John.14.2"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.14.2"
∷ word (μ ∷ ο ∷ ν ∷ α ∷ ὶ ∷ []) "John.14.2"
∷ word (π ∷ ο ∷ ∙λ ∷ ∙λ ∷ α ∷ ί ∷ []) "John.14.2"
∷ word (ε ∷ ἰ ∷ σ ∷ ι ∷ ν ∷ []) "John.14.2"
∷ word (ε ∷ ἰ ∷ []) "John.14.2"
∷ word (δ ∷ ὲ ∷ []) "John.14.2"
∷ word (μ ∷ ή ∷ []) "John.14.2"
∷ word (ε ∷ ἶ ∷ π ∷ ο ∷ ν ∷ []) "John.14.2"
∷ word (ἂ ∷ ν ∷ []) "John.14.2"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.14.2"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.14.2"
∷ word (π ∷ ο ∷ ρ ∷ ε ∷ ύ ∷ ο ∷ μ ∷ α ∷ ι ∷ []) "John.14.2"
∷ word (ἑ ∷ τ ∷ ο ∷ ι ∷ μ ∷ ά ∷ σ ∷ α ∷ ι ∷ []) "John.14.2"
∷ word (τ ∷ ό ∷ π ∷ ο ∷ ν ∷ []) "John.14.2"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.14.2"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.14.3"
∷ word (ἐ ∷ ὰ ∷ ν ∷ []) "John.14.3"
∷ word (π ∷ ο ∷ ρ ∷ ε ∷ υ ∷ θ ∷ ῶ ∷ []) "John.14.3"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.14.3"
∷ word (ἑ ∷ τ ∷ ο ∷ ι ∷ μ ∷ ά ∷ σ ∷ ω ∷ []) "John.14.3"
∷ word (τ ∷ ό ∷ π ∷ ο ∷ ν ∷ []) "John.14.3"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.14.3"
∷ word (π ∷ ά ∷ ∙λ ∷ ι ∷ ν ∷ []) "John.14.3"
∷ word (ἔ ∷ ρ ∷ χ ∷ ο ∷ μ ∷ α ∷ ι ∷ []) "John.14.3"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.14.3"
∷ word (π ∷ α ∷ ρ ∷ α ∷ ∙λ ∷ ή ∷ μ ∷ ψ ∷ ο ∷ μ ∷ α ∷ ι ∷ []) "John.14.3"
∷ word (ὑ ∷ μ ∷ ᾶ ∷ ς ∷ []) "John.14.3"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.14.3"
∷ word (ἐ ∷ μ ∷ α ∷ υ ∷ τ ∷ ό ∷ ν ∷ []) "John.14.3"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.14.3"
∷ word (ὅ ∷ π ∷ ο ∷ υ ∷ []) "John.14.3"
∷ word (ε ∷ ἰ ∷ μ ∷ ὶ ∷ []) "John.14.3"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.14.3"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.14.3"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.14.3"
∷ word (ἦ ∷ τ ∷ ε ∷ []) "John.14.3"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.14.4"
∷ word (ὅ ∷ π ∷ ο ∷ υ ∷ []) "John.14.4"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.14.4"
∷ word (ὑ ∷ π ∷ ά ∷ γ ∷ ω ∷ []) "John.14.4"
∷ word (ο ∷ ἴ ∷ δ ∷ α ∷ τ ∷ ε ∷ []) "John.14.4"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.14.4"
∷ word (ὁ ∷ δ ∷ ό ∷ ν ∷ []) "John.14.4"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.14.5"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.14.5"
∷ word (Θ ∷ ω ∷ μ ∷ ᾶ ∷ ς ∷ []) "John.14.5"
∷ word (Κ ∷ ύ ∷ ρ ∷ ι ∷ ε ∷ []) "John.14.5"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.14.5"
∷ word (ο ∷ ἴ ∷ δ ∷ α ∷ μ ∷ ε ∷ ν ∷ []) "John.14.5"
∷ word (π ∷ ο ∷ ῦ ∷ []) "John.14.5"
∷ word (ὑ ∷ π ∷ ά ∷ γ ∷ ε ∷ ι ∷ ς ∷ []) "John.14.5"
∷ word (π ∷ ῶ ∷ ς ∷ []) "John.14.5"
∷ word (δ ∷ υ ∷ ν ∷ ά ∷ μ ∷ ε ∷ θ ∷ α ∷ []) "John.14.5"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.14.5"
∷ word (ὁ ∷ δ ∷ ὸ ∷ ν ∷ []) "John.14.5"
∷ word (ε ∷ ἰ ∷ δ ∷ έ ∷ ν ∷ α ∷ ι ∷ []) "John.14.5"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.14.6"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.14.6"
∷ word (ὁ ∷ []) "John.14.6"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.14.6"
∷ word (Ἐ ∷ γ ∷ ώ ∷ []) "John.14.6"
∷ word (ε ∷ ἰ ∷ μ ∷ ι ∷ []) "John.14.6"
∷ word (ἡ ∷ []) "John.14.6"
∷ word (ὁ ∷ δ ∷ ὸ ∷ ς ∷ []) "John.14.6"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.14.6"
∷ word (ἡ ∷ []) "John.14.6"
∷ word (ἀ ∷ ∙λ ∷ ή ∷ θ ∷ ε ∷ ι ∷ α ∷ []) "John.14.6"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.14.6"
∷ word (ἡ ∷ []) "John.14.6"
∷ word (ζ ∷ ω ∷ ή ∷ []) "John.14.6"
∷ word (ο ∷ ὐ ∷ δ ∷ ε ∷ ὶ ∷ ς ∷ []) "John.14.6"
∷ word (ἔ ∷ ρ ∷ χ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.14.6"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.14.6"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.14.6"
∷ word (π ∷ α ∷ τ ∷ έ ∷ ρ ∷ α ∷ []) "John.14.6"
∷ word (ε ∷ ἰ ∷ []) "John.14.6"
∷ word (μ ∷ ὴ ∷ []) "John.14.6"
∷ word (δ ∷ ι ∷ []) "John.14.6"
∷ word (ἐ ∷ μ ∷ ο ∷ ῦ ∷ []) "John.14.6"
∷ word (ε ∷ ἰ ∷ []) "John.14.7"
∷ word (ἐ ∷ γ ∷ ν ∷ ώ ∷ κ ∷ ε ∷ ι ∷ τ ∷ έ ∷ []) "John.14.7"
∷ word (μ ∷ ε ∷ []) "John.14.7"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.14.7"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.14.7"
∷ word (π ∷ α ∷ τ ∷ έ ∷ ρ ∷ α ∷ []) "John.14.7"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.14.7"
∷ word (ἂ ∷ ν ∷ []) "John.14.7"
∷ word (ᾔ ∷ δ ∷ ε ∷ ι ∷ τ ∷ ε ∷ []) "John.14.7"
∷ word (ἀ ∷ π ∷ []) "John.14.7"
∷ word (ἄ ∷ ρ ∷ τ ∷ ι ∷ []) "John.14.7"
∷ word (γ ∷ ι ∷ ν ∷ ώ ∷ σ ∷ κ ∷ ε ∷ τ ∷ ε ∷ []) "John.14.7"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.14.7"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.14.7"
∷ word (ἑ ∷ ω ∷ ρ ∷ ά ∷ κ ∷ α ∷ τ ∷ ε ∷ []) "John.14.7"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.14.7"
∷ word (Λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.14.8"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.14.8"
∷ word (Φ ∷ ί ∷ ∙λ ∷ ι ∷ π ∷ π ∷ ο ∷ ς ∷ []) "John.14.8"
∷ word (Κ ∷ ύ ∷ ρ ∷ ι ∷ ε ∷ []) "John.14.8"
∷ word (δ ∷ ε ∷ ῖ ∷ ξ ∷ ο ∷ ν ∷ []) "John.14.8"
∷ word (ἡ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.14.8"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.14.8"
∷ word (π ∷ α ∷ τ ∷ έ ∷ ρ ∷ α ∷ []) "John.14.8"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.14.8"
∷ word (ἀ ∷ ρ ∷ κ ∷ ε ∷ ῖ ∷ []) "John.14.8"
∷ word (ἡ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.14.8"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.14.9"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.14.9"
∷ word (ὁ ∷ []) "John.14.9"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.14.9"
∷ word (Τ ∷ ο ∷ σ ∷ ο ∷ ύ ∷ τ ∷ ῳ ∷ []) "John.14.9"
∷ word (χ ∷ ρ ∷ ό ∷ ν ∷ ῳ ∷ []) "John.14.9"
∷ word (μ ∷ ε ∷ θ ∷ []) "John.14.9"
∷ word (ὑ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.14.9"
∷ word (ε ∷ ἰ ∷ μ ∷ ι ∷ []) "John.14.9"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.14.9"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.14.9"
∷ word (ἔ ∷ γ ∷ ν ∷ ω ∷ κ ∷ ά ∷ ς ∷ []) "John.14.9"
∷ word (μ ∷ ε ∷ []) "John.14.9"
∷ word (Φ ∷ ί ∷ ∙λ ∷ ι ∷ π ∷ π ∷ ε ∷ []) "John.14.9"
∷ word (ὁ ∷ []) "John.14.9"
∷ word (ἑ ∷ ω ∷ ρ ∷ α ∷ κ ∷ ὼ ∷ ς ∷ []) "John.14.9"
∷ word (ἐ ∷ μ ∷ ὲ ∷ []) "John.14.9"
∷ word (ἑ ∷ ώ ∷ ρ ∷ α ∷ κ ∷ ε ∷ ν ∷ []) "John.14.9"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.14.9"
∷ word (π ∷ α ∷ τ ∷ έ ∷ ρ ∷ α ∷ []) "John.14.9"
∷ word (π ∷ ῶ ∷ ς ∷ []) "John.14.9"
∷ word (σ ∷ ὺ ∷ []) "John.14.9"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ ς ∷ []) "John.14.9"
∷ word (Δ ∷ ε ∷ ῖ ∷ ξ ∷ ο ∷ ν ∷ []) "John.14.9"
∷ word (ἡ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.14.9"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.14.9"
∷ word (π ∷ α ∷ τ ∷ έ ∷ ρ ∷ α ∷ []) "John.14.9"
∷ word (ο ∷ ὐ ∷ []) "John.14.10"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ ε ∷ ι ∷ ς ∷ []) "John.14.10"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.14.10"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.14.10"
∷ word (ἐ ∷ ν ∷ []) "John.14.10"
∷ word (τ ∷ ῷ ∷ []) "John.14.10"
∷ word (π ∷ α ∷ τ ∷ ρ ∷ ὶ ∷ []) "John.14.10"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.14.10"
∷ word (ὁ ∷ []) "John.14.10"
∷ word (π ∷ α ∷ τ ∷ ὴ ∷ ρ ∷ []) "John.14.10"
∷ word (ἐ ∷ ν ∷ []) "John.14.10"
∷ word (ἐ ∷ μ ∷ ο ∷ ί ∷ []) "John.14.10"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.14.10"
∷ word (τ ∷ ὰ ∷ []) "John.14.10"
∷ word (ῥ ∷ ή ∷ μ ∷ α ∷ τ ∷ α ∷ []) "John.14.10"
∷ word (ἃ ∷ []) "John.14.10"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.14.10"
∷ word (∙λ ∷ έ ∷ γ ∷ ω ∷ []) "John.14.10"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.14.10"
∷ word (ἀ ∷ π ∷ []) "John.14.10"
∷ word (ἐ ∷ μ ∷ α ∷ υ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.14.10"
∷ word (ο ∷ ὐ ∷ []) "John.14.10"
∷ word (∙λ ∷ α ∷ ∙λ ∷ ῶ ∷ []) "John.14.10"
∷ word (ὁ ∷ []) "John.14.10"
∷ word (δ ∷ ὲ ∷ []) "John.14.10"
∷ word (π ∷ α ∷ τ ∷ ὴ ∷ ρ ∷ []) "John.14.10"
∷ word (ἐ ∷ ν ∷ []) "John.14.10"
∷ word (ἐ ∷ μ ∷ ο ∷ ὶ ∷ []) "John.14.10"
∷ word (μ ∷ έ ∷ ν ∷ ω ∷ ν ∷ []) "John.14.10"
∷ word (π ∷ ο ∷ ι ∷ ε ∷ ῖ ∷ []) "John.14.10"
∷ word (τ ∷ ὰ ∷ []) "John.14.10"
∷ word (ἔ ∷ ρ ∷ γ ∷ α ∷ []) "John.14.10"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.14.10"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ ε ∷ τ ∷ έ ∷ []) "John.14.11"
∷ word (μ ∷ ο ∷ ι ∷ []) "John.14.11"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.14.11"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.14.11"
∷ word (ἐ ∷ ν ∷ []) "John.14.11"
∷ word (τ ∷ ῷ ∷ []) "John.14.11"
∷ word (π ∷ α ∷ τ ∷ ρ ∷ ὶ ∷ []) "John.14.11"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.14.11"
∷ word (ὁ ∷ []) "John.14.11"
∷ word (π ∷ α ∷ τ ∷ ὴ ∷ ρ ∷ []) "John.14.11"
∷ word (ἐ ∷ ν ∷ []) "John.14.11"
∷ word (ἐ ∷ μ ∷ ο ∷ ί ∷ []) "John.14.11"
∷ word (ε ∷ ἰ ∷ []) "John.14.11"
∷ word (δ ∷ ὲ ∷ []) "John.14.11"
∷ word (μ ∷ ή ∷ []) "John.14.11"
∷ word (δ ∷ ι ∷ ὰ ∷ []) "John.14.11"
∷ word (τ ∷ ὰ ∷ []) "John.14.11"
∷ word (ἔ ∷ ρ ∷ γ ∷ α ∷ []) "John.14.11"
∷ word (α ∷ ὐ ∷ τ ∷ ὰ ∷ []) "John.14.11"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ ε ∷ τ ∷ ε ∷ []) "John.14.11"
∷ word (ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.14.12"
∷ word (ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.14.12"
∷ word (∙λ ∷ έ ∷ γ ∷ ω ∷ []) "John.14.12"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.14.12"
∷ word (ὁ ∷ []) "John.14.12"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ ω ∷ ν ∷ []) "John.14.12"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.14.12"
∷ word (ἐ ∷ μ ∷ ὲ ∷ []) "John.14.12"
∷ word (τ ∷ ὰ ∷ []) "John.14.12"
∷ word (ἔ ∷ ρ ∷ γ ∷ α ∷ []) "John.14.12"
∷ word (ἃ ∷ []) "John.14.12"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.14.12"
∷ word (π ∷ ο ∷ ι ∷ ῶ ∷ []) "John.14.12"
∷ word (κ ∷ ἀ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ο ∷ ς ∷ []) "John.14.12"
∷ word (π ∷ ο ∷ ι ∷ ή ∷ σ ∷ ε ∷ ι ∷ []) "John.14.12"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.14.12"
∷ word (μ ∷ ε ∷ ί ∷ ζ ∷ ο ∷ ν ∷ α ∷ []) "John.14.12"
∷ word (τ ∷ ο ∷ ύ ∷ τ ∷ ω ∷ ν ∷ []) "John.14.12"
∷ word (π ∷ ο ∷ ι ∷ ή ∷ σ ∷ ε ∷ ι ∷ []) "John.14.12"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.14.12"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.14.12"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.14.12"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.14.12"
∷ word (π ∷ α ∷ τ ∷ έ ∷ ρ ∷ α ∷ []) "John.14.12"
∷ word (π ∷ ο ∷ ρ ∷ ε ∷ ύ ∷ ο ∷ μ ∷ α ∷ ι ∷ []) "John.14.12"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.14.13"
∷ word (ὅ ∷ []) "John.14.13"
∷ word (τ ∷ ι ∷ []) "John.14.13"
∷ word (ἂ ∷ ν ∷ []) "John.14.13"
∷ word (α ∷ ἰ ∷ τ ∷ ή ∷ σ ∷ η ∷ τ ∷ ε ∷ []) "John.14.13"
∷ word (ἐ ∷ ν ∷ []) "John.14.13"
∷ word (τ ∷ ῷ ∷ []) "John.14.13"
∷ word (ὀ ∷ ν ∷ ό ∷ μ ∷ α ∷ τ ∷ ί ∷ []) "John.14.13"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.14.13"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.14.13"
∷ word (π ∷ ο ∷ ι ∷ ή ∷ σ ∷ ω ∷ []) "John.14.13"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.14.13"
∷ word (δ ∷ ο ∷ ξ ∷ α ∷ σ ∷ θ ∷ ῇ ∷ []) "John.14.13"
∷ word (ὁ ∷ []) "John.14.13"
∷ word (π ∷ α ∷ τ ∷ ὴ ∷ ρ ∷ []) "John.14.13"
∷ word (ἐ ∷ ν ∷ []) "John.14.13"
∷ word (τ ∷ ῷ ∷ []) "John.14.13"
∷ word (υ ∷ ἱ ∷ ῷ ∷ []) "John.14.13"
∷ word (ἐ ∷ ά ∷ ν ∷ []) "John.14.14"
∷ word (τ ∷ ι ∷ []) "John.14.14"
∷ word (α ∷ ἰ ∷ τ ∷ ή ∷ σ ∷ η ∷ τ ∷ έ ∷ []) "John.14.14"
∷ word (μ ∷ ε ∷ []) "John.14.14"
∷ word (ἐ ∷ ν ∷ []) "John.14.14"
∷ word (τ ∷ ῷ ∷ []) "John.14.14"
∷ word (ὀ ∷ ν ∷ ό ∷ μ ∷ α ∷ τ ∷ ί ∷ []) "John.14.14"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.14.14"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.14.14"
∷ word (π ∷ ο ∷ ι ∷ ή ∷ σ ∷ ω ∷ []) "John.14.14"
∷ word (Ἐ ∷ ὰ ∷ ν ∷ []) "John.14.15"
∷ word (ἀ ∷ γ ∷ α ∷ π ∷ ᾶ ∷ τ ∷ έ ∷ []) "John.14.15"
∷ word (μ ∷ ε ∷ []) "John.14.15"
∷ word (τ ∷ ὰ ∷ ς ∷ []) "John.14.15"
∷ word (ἐ ∷ ν ∷ τ ∷ ο ∷ ∙λ ∷ ὰ ∷ ς ∷ []) "John.14.15"
∷ word (τ ∷ ὰ ∷ ς ∷ []) "John.14.15"
∷ word (ἐ ∷ μ ∷ ὰ ∷ ς ∷ []) "John.14.15"
∷ word (τ ∷ η ∷ ρ ∷ ή ∷ σ ∷ ε ∷ τ ∷ ε ∷ []) "John.14.15"
∷ word (κ ∷ ἀ ∷ γ ∷ ὼ ∷ []) "John.14.16"
∷ word (ἐ ∷ ρ ∷ ω ∷ τ ∷ ή ∷ σ ∷ ω ∷ []) "John.14.16"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.14.16"
∷ word (π ∷ α ∷ τ ∷ έ ∷ ρ ∷ α ∷ []) "John.14.16"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.14.16"
∷ word (ἄ ∷ ∙λ ∷ ∙λ ∷ ο ∷ ν ∷ []) "John.14.16"
∷ word (π ∷ α ∷ ρ ∷ ά ∷ κ ∷ ∙λ ∷ η ∷ τ ∷ ο ∷ ν ∷ []) "John.14.16"
∷ word (δ ∷ ώ ∷ σ ∷ ε ∷ ι ∷ []) "John.14.16"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.14.16"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.14.16"
∷ word (ᾖ ∷ []) "John.14.16"
∷ word (μ ∷ ε ∷ θ ∷ []) "John.14.16"
∷ word (ὑ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.14.16"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.14.16"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.14.16"
∷ word (α ∷ ἰ ∷ ῶ ∷ ν ∷ α ∷ []) "John.14.16"
∷ word (τ ∷ ὸ ∷ []) "John.14.17"
∷ word (π ∷ ν ∷ ε ∷ ῦ ∷ μ ∷ α ∷ []) "John.14.17"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.14.17"
∷ word (ἀ ∷ ∙λ ∷ η ∷ θ ∷ ε ∷ ί ∷ α ∷ ς ∷ []) "John.14.17"
∷ word (ὃ ∷ []) "John.14.17"
∷ word (ὁ ∷ []) "John.14.17"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ ς ∷ []) "John.14.17"
∷ word (ο ∷ ὐ ∷ []) "John.14.17"
∷ word (δ ∷ ύ ∷ ν ∷ α ∷ τ ∷ α ∷ ι ∷ []) "John.14.17"
∷ word (∙λ ∷ α ∷ β ∷ ε ∷ ῖ ∷ ν ∷ []) "John.14.17"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.14.17"
∷ word (ο ∷ ὐ ∷ []) "John.14.17"
∷ word (θ ∷ ε ∷ ω ∷ ρ ∷ ε ∷ ῖ ∷ []) "John.14.17"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ []) "John.14.17"
∷ word (ο ∷ ὐ ∷ δ ∷ ὲ ∷ []) "John.14.17"
∷ word (γ ∷ ι ∷ ν ∷ ώ ∷ σ ∷ κ ∷ ε ∷ ι ∷ []) "John.14.17"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.14.17"
∷ word (γ ∷ ι ∷ ν ∷ ώ ∷ σ ∷ κ ∷ ε ∷ τ ∷ ε ∷ []) "John.14.17"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ []) "John.14.17"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.14.17"
∷ word (π ∷ α ∷ ρ ∷ []) "John.14.17"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.14.17"
∷ word (μ ∷ έ ∷ ν ∷ ε ∷ ι ∷ []) "John.14.17"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.14.17"
∷ word (ἐ ∷ ν ∷ []) "John.14.17"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.14.17"
∷ word (ἔ ∷ σ ∷ τ ∷ α ∷ ι ∷ []) "John.14.17"
∷ word (Ο ∷ ὐ ∷ κ ∷ []) "John.14.18"
∷ word (ἀ ∷ φ ∷ ή ∷ σ ∷ ω ∷ []) "John.14.18"
∷ word (ὑ ∷ μ ∷ ᾶ ∷ ς ∷ []) "John.14.18"
∷ word (ὀ ∷ ρ ∷ φ ∷ α ∷ ν ∷ ο ∷ ύ ∷ ς ∷ []) "John.14.18"
∷ word (ἔ ∷ ρ ∷ χ ∷ ο ∷ μ ∷ α ∷ ι ∷ []) "John.14.18"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.14.18"
∷ word (ὑ ∷ μ ∷ ᾶ ∷ ς ∷ []) "John.14.18"
∷ word (ἔ ∷ τ ∷ ι ∷ []) "John.14.19"
∷ word (μ ∷ ι ∷ κ ∷ ρ ∷ ὸ ∷ ν ∷ []) "John.14.19"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.14.19"
∷ word (ὁ ∷ []) "John.14.19"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ ς ∷ []) "John.14.19"
∷ word (μ ∷ ε ∷ []) "John.14.19"
∷ word (ο ∷ ὐ ∷ κ ∷ έ ∷ τ ∷ ι ∷ []) "John.14.19"
∷ word (θ ∷ ε ∷ ω ∷ ρ ∷ ε ∷ ῖ ∷ []) "John.14.19"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.14.19"
∷ word (δ ∷ ὲ ∷ []) "John.14.19"
∷ word (θ ∷ ε ∷ ω ∷ ρ ∷ ε ∷ ῖ ∷ τ ∷ έ ∷ []) "John.14.19"
∷ word (μ ∷ ε ∷ []) "John.14.19"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.14.19"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.14.19"
∷ word (ζ ∷ ῶ ∷ []) "John.14.19"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.14.19"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.14.19"
∷ word (ζ ∷ ή ∷ σ ∷ ε ∷ τ ∷ ε ∷ []) "John.14.19"
∷ word (ἐ ∷ ν ∷ []) "John.14.20"
∷ word (ἐ ∷ κ ∷ ε ∷ ί ∷ ν ∷ ῃ ∷ []) "John.14.20"
∷ word (τ ∷ ῇ ∷ []) "John.14.20"
∷ word (ἡ ∷ μ ∷ έ ∷ ρ ∷ ᾳ ∷ []) "John.14.20"
∷ word (γ ∷ ν ∷ ώ ∷ σ ∷ ε ∷ σ ∷ θ ∷ ε ∷ []) "John.14.20"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.14.20"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.14.20"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.14.20"
∷ word (ἐ ∷ ν ∷ []) "John.14.20"
∷ word (τ ∷ ῷ ∷ []) "John.14.20"
∷ word (π ∷ α ∷ τ ∷ ρ ∷ ί ∷ []) "John.14.20"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.14.20"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.14.20"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.14.20"
∷ word (ἐ ∷ ν ∷ []) "John.14.20"
∷ word (ἐ ∷ μ ∷ ο ∷ ὶ ∷ []) "John.14.20"
∷ word (κ ∷ ἀ ∷ γ ∷ ὼ ∷ []) "John.14.20"
∷ word (ἐ ∷ ν ∷ []) "John.14.20"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.14.20"
∷ word (ὁ ∷ []) "John.14.21"
∷ word (ἔ ∷ χ ∷ ω ∷ ν ∷ []) "John.14.21"
∷ word (τ ∷ ὰ ∷ ς ∷ []) "John.14.21"
∷ word (ἐ ∷ ν ∷ τ ∷ ο ∷ ∙λ ∷ ά ∷ ς ∷ []) "John.14.21"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.14.21"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.14.21"
∷ word (τ ∷ η ∷ ρ ∷ ῶ ∷ ν ∷ []) "John.14.21"
∷ word (α ∷ ὐ ∷ τ ∷ ὰ ∷ ς ∷ []) "John.14.21"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ό ∷ ς ∷ []) "John.14.21"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.14.21"
∷ word (ὁ ∷ []) "John.14.21"
∷ word (ἀ ∷ γ ∷ α ∷ π ∷ ῶ ∷ ν ∷ []) "John.14.21"
∷ word (μ ∷ ε ∷ []) "John.14.21"
∷ word (ὁ ∷ []) "John.14.21"
∷ word (δ ∷ ὲ ∷ []) "John.14.21"
∷ word (ἀ ∷ γ ∷ α ∷ π ∷ ῶ ∷ ν ∷ []) "John.14.21"
∷ word (μ ∷ ε ∷ []) "John.14.21"
∷ word (ἀ ∷ γ ∷ α ∷ π ∷ η ∷ θ ∷ ή ∷ σ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.14.21"
∷ word (ὑ ∷ π ∷ ὸ ∷ []) "John.14.21"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.14.21"
∷ word (π ∷ α ∷ τ ∷ ρ ∷ ό ∷ ς ∷ []) "John.14.21"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.14.21"
∷ word (κ ∷ ἀ ∷ γ ∷ ὼ ∷ []) "John.14.21"
∷ word (ἀ ∷ γ ∷ α ∷ π ∷ ή ∷ σ ∷ ω ∷ []) "John.14.21"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.14.21"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.14.21"
∷ word (ἐ ∷ μ ∷ φ ∷ α ∷ ν ∷ ί ∷ σ ∷ ω ∷ []) "John.14.21"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.14.21"
∷ word (ἐ ∷ μ ∷ α ∷ υ ∷ τ ∷ ό ∷ ν ∷ []) "John.14.21"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.14.22"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.14.22"
∷ word (Ἰ ∷ ο ∷ ύ ∷ δ ∷ α ∷ ς ∷ []) "John.14.22"
∷ word (ο ∷ ὐ ∷ χ ∷ []) "John.14.22"
∷ word (ὁ ∷ []) "John.14.22"
∷ word (Ἰ ∷ σ ∷ κ ∷ α ∷ ρ ∷ ι ∷ ώ ∷ τ ∷ η ∷ ς ∷ []) "John.14.22"
∷ word (Κ ∷ ύ ∷ ρ ∷ ι ∷ ε ∷ []) "John.14.22"
∷ word (τ ∷ ί ∷ []) "John.14.22"
∷ word (γ ∷ έ ∷ γ ∷ ο ∷ ν ∷ ε ∷ ν ∷ []) "John.14.22"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.14.22"
∷ word (ἡ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.14.22"
∷ word (μ ∷ έ ∷ ∙λ ∷ ∙λ ∷ ε ∷ ι ∷ ς ∷ []) "John.14.22"
∷ word (ἐ ∷ μ ∷ φ ∷ α ∷ ν ∷ ί ∷ ζ ∷ ε ∷ ι ∷ ν ∷ []) "John.14.22"
∷ word (σ ∷ ε ∷ α ∷ υ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.14.22"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.14.22"
∷ word (ο ∷ ὐ ∷ χ ∷ ὶ ∷ []) "John.14.22"
∷ word (τ ∷ ῷ ∷ []) "John.14.22"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ῳ ∷ []) "John.14.22"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.14.23"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.14.23"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.14.23"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.14.23"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.14.23"
∷ word (Ἐ ∷ ά ∷ ν ∷ []) "John.14.23"
∷ word (τ ∷ ι ∷ ς ∷ []) "John.14.23"
∷ word (ἀ ∷ γ ∷ α ∷ π ∷ ᾷ ∷ []) "John.14.23"
∷ word (μ ∷ ε ∷ []) "John.14.23"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.14.23"
∷ word (∙λ ∷ ό ∷ γ ∷ ο ∷ ν ∷ []) "John.14.23"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.14.23"
∷ word (τ ∷ η ∷ ρ ∷ ή ∷ σ ∷ ε ∷ ι ∷ []) "John.14.23"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.14.23"
∷ word (ὁ ∷ []) "John.14.23"
∷ word (π ∷ α ∷ τ ∷ ή ∷ ρ ∷ []) "John.14.23"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.14.23"
∷ word (ἀ ∷ γ ∷ α ∷ π ∷ ή ∷ σ ∷ ε ∷ ι ∷ []) "John.14.23"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.14.23"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.14.23"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.14.23"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.14.23"
∷ word (ἐ ∷ ∙λ ∷ ε ∷ υ ∷ σ ∷ ό ∷ μ ∷ ε ∷ θ ∷ α ∷ []) "John.14.23"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.14.23"
∷ word (μ ∷ ο ∷ ν ∷ ὴ ∷ ν ∷ []) "John.14.23"
∷ word (π ∷ α ∷ ρ ∷ []) "John.14.23"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.14.23"
∷ word (π ∷ ο ∷ ι ∷ η ∷ σ ∷ ό ∷ μ ∷ ε ∷ θ ∷ α ∷ []) "John.14.23"
∷ word (ὁ ∷ []) "John.14.24"
∷ word (μ ∷ ὴ ∷ []) "John.14.24"
∷ word (ἀ ∷ γ ∷ α ∷ π ∷ ῶ ∷ ν ∷ []) "John.14.24"
∷ word (μ ∷ ε ∷ []) "John.14.24"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.14.24"
∷ word (∙λ ∷ ό ∷ γ ∷ ο ∷ υ ∷ ς ∷ []) "John.14.24"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.14.24"
∷ word (ο ∷ ὐ ∷ []) "John.14.24"
∷ word (τ ∷ η ∷ ρ ∷ ε ∷ ῖ ∷ []) "John.14.24"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.14.24"
∷ word (ὁ ∷ []) "John.14.24"
∷ word (∙λ ∷ ό ∷ γ ∷ ο ∷ ς ∷ []) "John.14.24"
∷ word (ὃ ∷ ν ∷ []) "John.14.24"
∷ word (ἀ ∷ κ ∷ ο ∷ ύ ∷ ε ∷ τ ∷ ε ∷ []) "John.14.24"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.14.24"
∷ word (ἔ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.14.24"
∷ word (ἐ ∷ μ ∷ ὸ ∷ ς ∷ []) "John.14.24"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.14.24"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.14.24"
∷ word (π ∷ έ ∷ μ ∷ ψ ∷ α ∷ ν ∷ τ ∷ ό ∷ ς ∷ []) "John.14.24"
∷ word (μ ∷ ε ∷ []) "John.14.24"
∷ word (π ∷ α ∷ τ ∷ ρ ∷ ό ∷ ς ∷ []) "John.14.24"
∷ word (Τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.14.25"
∷ word (∙λ ∷ ε ∷ ∙λ ∷ ά ∷ ∙λ ∷ η ∷ κ ∷ α ∷ []) "John.14.25"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.14.25"
∷ word (π ∷ α ∷ ρ ∷ []) "John.14.25"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.14.25"
∷ word (μ ∷ έ ∷ ν ∷ ω ∷ ν ∷ []) "John.14.25"
∷ word (ὁ ∷ []) "John.14.26"
∷ word (δ ∷ ὲ ∷ []) "John.14.26"
∷ word (π ∷ α ∷ ρ ∷ ά ∷ κ ∷ ∙λ ∷ η ∷ τ ∷ ο ∷ ς ∷ []) "John.14.26"
∷ word (τ ∷ ὸ ∷ []) "John.14.26"
∷ word (π ∷ ν ∷ ε ∷ ῦ ∷ μ ∷ α ∷ []) "John.14.26"
∷ word (τ ∷ ὸ ∷ []) "John.14.26"
∷ word (ἅ ∷ γ ∷ ι ∷ ο ∷ ν ∷ []) "John.14.26"
∷ word (ὃ ∷ []) "John.14.26"
∷ word (π ∷ έ ∷ μ ∷ ψ ∷ ε ∷ ι ∷ []) "John.14.26"
∷ word (ὁ ∷ []) "John.14.26"
∷ word (π ∷ α ∷ τ ∷ ὴ ∷ ρ ∷ []) "John.14.26"
∷ word (ἐ ∷ ν ∷ []) "John.14.26"
∷ word (τ ∷ ῷ ∷ []) "John.14.26"
∷ word (ὀ ∷ ν ∷ ό ∷ μ ∷ α ∷ τ ∷ ί ∷ []) "John.14.26"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.14.26"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ο ∷ ς ∷ []) "John.14.26"
∷ word (ὑ ∷ μ ∷ ᾶ ∷ ς ∷ []) "John.14.26"
∷ word (δ ∷ ι ∷ δ ∷ ά ∷ ξ ∷ ε ∷ ι ∷ []) "John.14.26"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ α ∷ []) "John.14.26"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.14.26"
∷ word (ὑ ∷ π ∷ ο ∷ μ ∷ ν ∷ ή ∷ σ ∷ ε ∷ ι ∷ []) "John.14.26"
∷ word (ὑ ∷ μ ∷ ᾶ ∷ ς ∷ []) "John.14.26"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ α ∷ []) "John.14.26"
∷ word (ἃ ∷ []) "John.14.26"
∷ word (ε ∷ ἶ ∷ π ∷ ο ∷ ν ∷ []) "John.14.26"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.14.26"
∷ word (ε ∷ ἰ ∷ ρ ∷ ή ∷ ν ∷ η ∷ ν ∷ []) "John.14.27"
∷ word (ἀ ∷ φ ∷ ί ∷ η ∷ μ ∷ ι ∷ []) "John.14.27"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.14.27"
∷ word (ε ∷ ἰ ∷ ρ ∷ ή ∷ ν ∷ η ∷ ν ∷ []) "John.14.27"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.14.27"
∷ word (ἐ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.14.27"
∷ word (δ ∷ ί ∷ δ ∷ ω ∷ μ ∷ ι ∷ []) "John.14.27"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.14.27"
∷ word (ο ∷ ὐ ∷ []) "John.14.27"
∷ word (κ ∷ α ∷ θ ∷ ὼ ∷ ς ∷ []) "John.14.27"
∷ word (ὁ ∷ []) "John.14.27"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ ς ∷ []) "John.14.27"
∷ word (δ ∷ ί ∷ δ ∷ ω ∷ σ ∷ ι ∷ ν ∷ []) "John.14.27"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.14.27"
∷ word (δ ∷ ί ∷ δ ∷ ω ∷ μ ∷ ι ∷ []) "John.14.27"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.14.27"
∷ word (μ ∷ ὴ ∷ []) "John.14.27"
∷ word (τ ∷ α ∷ ρ ∷ α ∷ σ ∷ σ ∷ έ ∷ σ ∷ θ ∷ ω ∷ []) "John.14.27"
∷ word (ὑ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.14.27"
∷ word (ἡ ∷ []) "John.14.27"
∷ word (κ ∷ α ∷ ρ ∷ δ ∷ ί ∷ α ∷ []) "John.14.27"
∷ word (μ ∷ η ∷ δ ∷ ὲ ∷ []) "John.14.27"
∷ word (δ ∷ ε ∷ ι ∷ ∙λ ∷ ι ∷ ά ∷ τ ∷ ω ∷ []) "John.14.27"
∷ word (ἠ ∷ κ ∷ ο ∷ ύ ∷ σ ∷ α ∷ τ ∷ ε ∷ []) "John.14.28"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.14.28"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.14.28"
∷ word (ε ∷ ἶ ∷ π ∷ ο ∷ ν ∷ []) "John.14.28"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.14.28"
∷ word (Ὑ ∷ π ∷ ά ∷ γ ∷ ω ∷ []) "John.14.28"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.14.28"
∷ word (ἔ ∷ ρ ∷ χ ∷ ο ∷ μ ∷ α ∷ ι ∷ []) "John.14.28"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.14.28"
∷ word (ὑ ∷ μ ∷ ᾶ ∷ ς ∷ []) "John.14.28"
∷ word (ε ∷ ἰ ∷ []) "John.14.28"
∷ word (ἠ ∷ γ ∷ α ∷ π ∷ ᾶ ∷ τ ∷ έ ∷ []) "John.14.28"
∷ word (μ ∷ ε ∷ []) "John.14.28"
∷ word (ἐ ∷ χ ∷ ά ∷ ρ ∷ η ∷ τ ∷ ε ∷ []) "John.14.28"
∷ word (ἄ ∷ ν ∷ []) "John.14.28"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.14.28"
∷ word (π ∷ ο ∷ ρ ∷ ε ∷ ύ ∷ ο ∷ μ ∷ α ∷ ι ∷ []) "John.14.28"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.14.28"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.14.28"
∷ word (π ∷ α ∷ τ ∷ έ ∷ ρ ∷ α ∷ []) "John.14.28"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.14.28"
∷ word (ὁ ∷ []) "John.14.28"
∷ word (π ∷ α ∷ τ ∷ ὴ ∷ ρ ∷ []) "John.14.28"
∷ word (μ ∷ ε ∷ ί ∷ ζ ∷ ω ∷ ν ∷ []) "John.14.28"
∷ word (μ ∷ ο ∷ ύ ∷ []) "John.14.28"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.14.28"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.14.29"
∷ word (ν ∷ ῦ ∷ ν ∷ []) "John.14.29"
∷ word (ε ∷ ἴ ∷ ρ ∷ η ∷ κ ∷ α ∷ []) "John.14.29"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.14.29"
∷ word (π ∷ ρ ∷ ὶ ∷ ν ∷ []) "John.14.29"
∷ word (γ ∷ ε ∷ ν ∷ έ ∷ σ ∷ θ ∷ α ∷ ι ∷ []) "John.14.29"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.14.29"
∷ word (ὅ ∷ τ ∷ α ∷ ν ∷ []) "John.14.29"
∷ word (γ ∷ έ ∷ ν ∷ η ∷ τ ∷ α ∷ ι ∷ []) "John.14.29"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ σ ∷ η ∷ τ ∷ ε ∷ []) "John.14.29"
∷ word (ο ∷ ὐ ∷ κ ∷ έ ∷ τ ∷ ι ∷ []) "John.14.30"
∷ word (π ∷ ο ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.14.30"
∷ word (∙λ ∷ α ∷ ∙λ ∷ ή ∷ σ ∷ ω ∷ []) "John.14.30"
∷ word (μ ∷ ε ∷ θ ∷ []) "John.14.30"
∷ word (ὑ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.14.30"
∷ word (ἔ ∷ ρ ∷ χ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.14.30"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.14.30"
∷ word (ὁ ∷ []) "John.14.30"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.14.30"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ υ ∷ []) "John.14.30"
∷ word (ἄ ∷ ρ ∷ χ ∷ ω ∷ ν ∷ []) "John.14.30"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.14.30"
∷ word (ἐ ∷ ν ∷ []) "John.14.30"
∷ word (ἐ ∷ μ ∷ ο ∷ ὶ ∷ []) "John.14.30"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.14.30"
∷ word (ἔ ∷ χ ∷ ε ∷ ι ∷ []) "John.14.30"
∷ word (ο ∷ ὐ ∷ δ ∷ έ ∷ ν ∷ []) "John.14.30"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ []) "John.14.31"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.14.31"
∷ word (γ ∷ ν ∷ ῷ ∷ []) "John.14.31"
∷ word (ὁ ∷ []) "John.14.31"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ ς ∷ []) "John.14.31"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.14.31"
∷ word (ἀ ∷ γ ∷ α ∷ π ∷ ῶ ∷ []) "John.14.31"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.14.31"
∷ word (π ∷ α ∷ τ ∷ έ ∷ ρ ∷ α ∷ []) "John.14.31"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.14.31"
∷ word (κ ∷ α ∷ θ ∷ ὼ ∷ ς ∷ []) "John.14.31"
∷ word (ἐ ∷ ν ∷ ε ∷ τ ∷ ε ∷ ί ∷ ∙λ ∷ α ∷ τ ∷ ο ∷ []) "John.14.31"
∷ word (μ ∷ ο ∷ ι ∷ []) "John.14.31"
∷ word (ὁ ∷ []) "John.14.31"
∷ word (π ∷ α ∷ τ ∷ ὴ ∷ ρ ∷ []) "John.14.31"
∷ word (ο ∷ ὕ ∷ τ ∷ ω ∷ ς ∷ []) "John.14.31"
∷ word (π ∷ ο ∷ ι ∷ ῶ ∷ []) "John.14.31"
∷ word (Ἐ ∷ γ ∷ ε ∷ ί ∷ ρ ∷ ε ∷ σ ∷ θ ∷ ε ∷ []) "John.14.31"
∷ word (ἄ ∷ γ ∷ ω ∷ μ ∷ ε ∷ ν ∷ []) "John.14.31"
∷ word (ἐ ∷ ν ∷ τ ∷ ε ∷ ῦ ∷ θ ∷ ε ∷ ν ∷ []) "John.14.31"
∷ word (Ἐ ∷ γ ∷ ώ ∷ []) "John.15.1"
∷ word (ε ∷ ἰ ∷ μ ∷ ι ∷ []) "John.15.1"
∷ word (ἡ ∷ []) "John.15.1"
∷ word (ἄ ∷ μ ∷ π ∷ ε ∷ ∙λ ∷ ο ∷ ς ∷ []) "John.15.1"
∷ word (ἡ ∷ []) "John.15.1"
∷ word (ἀ ∷ ∙λ ∷ η ∷ θ ∷ ι ∷ ν ∷ ή ∷ []) "John.15.1"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.15.1"
∷ word (ὁ ∷ []) "John.15.1"
∷ word (π ∷ α ∷ τ ∷ ή ∷ ρ ∷ []) "John.15.1"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.15.1"
∷ word (ὁ ∷ []) "John.15.1"
∷ word (γ ∷ ε ∷ ω ∷ ρ ∷ γ ∷ ό ∷ ς ∷ []) "John.15.1"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.15.1"
∷ word (π ∷ ᾶ ∷ ν ∷ []) "John.15.2"
∷ word (κ ∷ ∙λ ∷ ῆ ∷ μ ∷ α ∷ []) "John.15.2"
∷ word (ἐ ∷ ν ∷ []) "John.15.2"
∷ word (ἐ ∷ μ ∷ ο ∷ ὶ ∷ []) "John.15.2"
∷ word (μ ∷ ὴ ∷ []) "John.15.2"
∷ word (φ ∷ έ ∷ ρ ∷ ο ∷ ν ∷ []) "John.15.2"
∷ word (κ ∷ α ∷ ρ ∷ π ∷ ὸ ∷ ν ∷ []) "John.15.2"
∷ word (α ∷ ἴ ∷ ρ ∷ ε ∷ ι ∷ []) "John.15.2"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ []) "John.15.2"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.15.2"
∷ word (π ∷ ᾶ ∷ ν ∷ []) "John.15.2"
∷ word (τ ∷ ὸ ∷ []) "John.15.2"
∷ word (κ ∷ α ∷ ρ ∷ π ∷ ὸ ∷ ν ∷ []) "John.15.2"
∷ word (φ ∷ έ ∷ ρ ∷ ο ∷ ν ∷ []) "John.15.2"
∷ word (κ ∷ α ∷ θ ∷ α ∷ ί ∷ ρ ∷ ε ∷ ι ∷ []) "John.15.2"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ []) "John.15.2"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.15.2"
∷ word (κ ∷ α ∷ ρ ∷ π ∷ ὸ ∷ ν ∷ []) "John.15.2"
∷ word (π ∷ ∙λ ∷ ε ∷ ί ∷ ο ∷ ν ∷ α ∷ []) "John.15.2"
∷ word (φ ∷ έ ∷ ρ ∷ ῃ ∷ []) "John.15.2"
∷ word (ἤ ∷ δ ∷ η ∷ []) "John.15.3"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.15.3"
∷ word (κ ∷ α ∷ θ ∷ α ∷ ρ ∷ ο ∷ ί ∷ []) "John.15.3"
∷ word (ἐ ∷ σ ∷ τ ∷ ε ∷ []) "John.15.3"
∷ word (δ ∷ ι ∷ ὰ ∷ []) "John.15.3"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.15.3"
∷ word (∙λ ∷ ό ∷ γ ∷ ο ∷ ν ∷ []) "John.15.3"
∷ word (ὃ ∷ ν ∷ []) "John.15.3"
∷ word (∙λ ∷ ε ∷ ∙λ ∷ ά ∷ ∙λ ∷ η ∷ κ ∷ α ∷ []) "John.15.3"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.15.3"
∷ word (μ ∷ ε ∷ ί ∷ ν ∷ α ∷ τ ∷ ε ∷ []) "John.15.4"
∷ word (ἐ ∷ ν ∷ []) "John.15.4"
∷ word (ἐ ∷ μ ∷ ο ∷ ί ∷ []) "John.15.4"
∷ word (κ ∷ ἀ ∷ γ ∷ ὼ ∷ []) "John.15.4"
∷ word (ἐ ∷ ν ∷ []) "John.15.4"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.15.4"
∷ word (κ ∷ α ∷ θ ∷ ὼ ∷ ς ∷ []) "John.15.4"
∷ word (τ ∷ ὸ ∷ []) "John.15.4"
∷ word (κ ∷ ∙λ ∷ ῆ ∷ μ ∷ α ∷ []) "John.15.4"
∷ word (ο ∷ ὐ ∷ []) "John.15.4"
∷ word (δ ∷ ύ ∷ ν ∷ α ∷ τ ∷ α ∷ ι ∷ []) "John.15.4"
∷ word (κ ∷ α ∷ ρ ∷ π ∷ ὸ ∷ ν ∷ []) "John.15.4"
∷ word (φ ∷ έ ∷ ρ ∷ ε ∷ ι ∷ ν ∷ []) "John.15.4"
∷ word (ἀ ∷ φ ∷ []) "John.15.4"
∷ word (ἑ ∷ α ∷ υ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.15.4"
∷ word (ἐ ∷ ὰ ∷ ν ∷ []) "John.15.4"
∷ word (μ ∷ ὴ ∷ []) "John.15.4"
∷ word (μ ∷ έ ∷ ν ∷ ῃ ∷ []) "John.15.4"
∷ word (ἐ ∷ ν ∷ []) "John.15.4"
∷ word (τ ∷ ῇ ∷ []) "John.15.4"
∷ word (ἀ ∷ μ ∷ π ∷ έ ∷ ∙λ ∷ ῳ ∷ []) "John.15.4"
∷ word (ο ∷ ὕ ∷ τ ∷ ω ∷ ς ∷ []) "John.15.4"
∷ word (ο ∷ ὐ ∷ δ ∷ ὲ ∷ []) "John.15.4"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.15.4"
∷ word (ἐ ∷ ὰ ∷ ν ∷ []) "John.15.4"
∷ word (μ ∷ ὴ ∷ []) "John.15.4"
∷ word (ἐ ∷ ν ∷ []) "John.15.4"
∷ word (ἐ ∷ μ ∷ ο ∷ ὶ ∷ []) "John.15.4"
∷ word (μ ∷ έ ∷ ν ∷ η ∷ τ ∷ ε ∷ []) "John.15.4"
∷ word (ἐ ∷ γ ∷ ώ ∷ []) "John.15.5"
∷ word (ε ∷ ἰ ∷ μ ∷ ι ∷ []) "John.15.5"
∷ word (ἡ ∷ []) "John.15.5"
∷ word (ἄ ∷ μ ∷ π ∷ ε ∷ ∙λ ∷ ο ∷ ς ∷ []) "John.15.5"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.15.5"
∷ word (τ ∷ ὰ ∷ []) "John.15.5"
∷ word (κ ∷ ∙λ ∷ ή ∷ μ ∷ α ∷ τ ∷ α ∷ []) "John.15.5"
∷ word (ὁ ∷ []) "John.15.5"
∷ word (μ ∷ έ ∷ ν ∷ ω ∷ ν ∷ []) "John.15.5"
∷ word (ἐ ∷ ν ∷ []) "John.15.5"
∷ word (ἐ ∷ μ ∷ ο ∷ ὶ ∷ []) "John.15.5"
∷ word (κ ∷ ἀ ∷ γ ∷ ὼ ∷ []) "John.15.5"
∷ word (ἐ ∷ ν ∷ []) "John.15.5"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.15.5"
∷ word (ο ∷ ὗ ∷ τ ∷ ο ∷ ς ∷ []) "John.15.5"
∷ word (φ ∷ έ ∷ ρ ∷ ε ∷ ι ∷ []) "John.15.5"
∷ word (κ ∷ α ∷ ρ ∷ π ∷ ὸ ∷ ν ∷ []) "John.15.5"
∷ word (π ∷ ο ∷ ∙λ ∷ ύ ∷ ν ∷ []) "John.15.5"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.15.5"
∷ word (χ ∷ ω ∷ ρ ∷ ὶ ∷ ς ∷ []) "John.15.5"
∷ word (ἐ ∷ μ ∷ ο ∷ ῦ ∷ []) "John.15.5"
∷ word (ο ∷ ὐ ∷ []) "John.15.5"
∷ word (δ ∷ ύ ∷ ν ∷ α ∷ σ ∷ θ ∷ ε ∷ []) "John.15.5"
∷ word (π ∷ ο ∷ ι ∷ ε ∷ ῖ ∷ ν ∷ []) "John.15.5"
∷ word (ο ∷ ὐ ∷ δ ∷ έ ∷ ν ∷ []) "John.15.5"
∷ word (ἐ ∷ ὰ ∷ ν ∷ []) "John.15.6"
∷ word (μ ∷ ή ∷ []) "John.15.6"
∷ word (τ ∷ ι ∷ ς ∷ []) "John.15.6"
∷ word (μ ∷ έ ∷ ν ∷ ῃ ∷ []) "John.15.6"
∷ word (ἐ ∷ ν ∷ []) "John.15.6"
∷ word (ἐ ∷ μ ∷ ο ∷ ί ∷ []) "John.15.6"
∷ word (ἐ ∷ β ∷ ∙λ ∷ ή ∷ θ ∷ η ∷ []) "John.15.6"
∷ word (ἔ ∷ ξ ∷ ω ∷ []) "John.15.6"
∷ word (ὡ ∷ ς ∷ []) "John.15.6"
∷ word (τ ∷ ὸ ∷ []) "John.15.6"
∷ word (κ ∷ ∙λ ∷ ῆ ∷ μ ∷ α ∷ []) "John.15.6"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.15.6"
∷ word (ἐ ∷ ξ ∷ η ∷ ρ ∷ ά ∷ ν ∷ θ ∷ η ∷ []) "John.15.6"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.15.6"
∷ word (σ ∷ υ ∷ ν ∷ ά ∷ γ ∷ ο ∷ υ ∷ σ ∷ ι ∷ ν ∷ []) "John.15.6"
∷ word (α ∷ ὐ ∷ τ ∷ ὰ ∷ []) "John.15.6"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.15.6"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.15.6"
∷ word (τ ∷ ὸ ∷ []) "John.15.6"
∷ word (π ∷ ῦ ∷ ρ ∷ []) "John.15.6"
∷ word (β ∷ ά ∷ ∙λ ∷ ∙λ ∷ ο ∷ υ ∷ σ ∷ ι ∷ ν ∷ []) "John.15.6"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.15.6"
∷ word (κ ∷ α ∷ ί ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.15.6"
∷ word (ἐ ∷ ὰ ∷ ν ∷ []) "John.15.7"
∷ word (μ ∷ ε ∷ ί ∷ ν ∷ η ∷ τ ∷ ε ∷ []) "John.15.7"
∷ word (ἐ ∷ ν ∷ []) "John.15.7"
∷ word (ἐ ∷ μ ∷ ο ∷ ὶ ∷ []) "John.15.7"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.15.7"
∷ word (τ ∷ ὰ ∷ []) "John.15.7"
∷ word (ῥ ∷ ή ∷ μ ∷ α ∷ τ ∷ ά ∷ []) "John.15.7"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.15.7"
∷ word (ἐ ∷ ν ∷ []) "John.15.7"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.15.7"
∷ word (μ ∷ ε ∷ ί ∷ ν ∷ ῃ ∷ []) "John.15.7"
∷ word (ὃ ∷ []) "John.15.7"
∷ word (ἐ ∷ ὰ ∷ ν ∷ []) "John.15.7"
∷ word (θ ∷ έ ∷ ∙λ ∷ η ∷ τ ∷ ε ∷ []) "John.15.7"
∷ word (α ∷ ἰ ∷ τ ∷ ή ∷ σ ∷ α ∷ σ ∷ θ ∷ ε ∷ []) "John.15.7"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.15.7"
∷ word (γ ∷ ε ∷ ν ∷ ή ∷ σ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.15.7"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.15.7"
∷ word (ἐ ∷ ν ∷ []) "John.15.8"
∷ word (τ ∷ ο ∷ ύ ∷ τ ∷ ῳ ∷ []) "John.15.8"
∷ word (ἐ ∷ δ ∷ ο ∷ ξ ∷ ά ∷ σ ∷ θ ∷ η ∷ []) "John.15.8"
∷ word (ὁ ∷ []) "John.15.8"
∷ word (π ∷ α ∷ τ ∷ ή ∷ ρ ∷ []) "John.15.8"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.15.8"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.15.8"
∷ word (κ ∷ α ∷ ρ ∷ π ∷ ὸ ∷ ν ∷ []) "John.15.8"
∷ word (π ∷ ο ∷ ∙λ ∷ ὺ ∷ ν ∷ []) "John.15.8"
∷ word (φ ∷ έ ∷ ρ ∷ η ∷ τ ∷ ε ∷ []) "John.15.8"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.15.8"
∷ word (γ ∷ έ ∷ ν ∷ η ∷ σ ∷ θ ∷ ε ∷ []) "John.15.8"
∷ word (ἐ ∷ μ ∷ ο ∷ ὶ ∷ []) "John.15.8"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ α ∷ ί ∷ []) "John.15.8"
∷ word (κ ∷ α ∷ θ ∷ ὼ ∷ ς ∷ []) "John.15.9"
∷ word (ἠ ∷ γ ∷ ά ∷ π ∷ η ∷ σ ∷ έ ∷ ν ∷ []) "John.15.9"
∷ word (μ ∷ ε ∷ []) "John.15.9"
∷ word (ὁ ∷ []) "John.15.9"
∷ word (π ∷ α ∷ τ ∷ ή ∷ ρ ∷ []) "John.15.9"
∷ word (κ ∷ ἀ ∷ γ ∷ ὼ ∷ []) "John.15.9"
∷ word (ὑ ∷ μ ∷ ᾶ ∷ ς ∷ []) "John.15.9"
∷ word (ἠ ∷ γ ∷ ά ∷ π ∷ η ∷ σ ∷ α ∷ []) "John.15.9"
∷ word (μ ∷ ε ∷ ί ∷ ν ∷ α ∷ τ ∷ ε ∷ []) "John.15.9"
∷ word (ἐ ∷ ν ∷ []) "John.15.9"
∷ word (τ ∷ ῇ ∷ []) "John.15.9"
∷ word (ἀ ∷ γ ∷ ά ∷ π ∷ ῃ ∷ []) "John.15.9"
∷ word (τ ∷ ῇ ∷ []) "John.15.9"
∷ word (ἐ ∷ μ ∷ ῇ ∷ []) "John.15.9"
∷ word (ἐ ∷ ὰ ∷ ν ∷ []) "John.15.10"
∷ word (τ ∷ ὰ ∷ ς ∷ []) "John.15.10"
∷ word (ἐ ∷ ν ∷ τ ∷ ο ∷ ∙λ ∷ ά ∷ ς ∷ []) "John.15.10"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.15.10"
∷ word (τ ∷ η ∷ ρ ∷ ή ∷ σ ∷ η ∷ τ ∷ ε ∷ []) "John.15.10"
∷ word (μ ∷ ε ∷ ν ∷ ε ∷ ῖ ∷ τ ∷ ε ∷ []) "John.15.10"
∷ word (ἐ ∷ ν ∷ []) "John.15.10"
∷ word (τ ∷ ῇ ∷ []) "John.15.10"
∷ word (ἀ ∷ γ ∷ ά ∷ π ∷ ῃ ∷ []) "John.15.10"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.15.10"
∷ word (κ ∷ α ∷ θ ∷ ὼ ∷ ς ∷ []) "John.15.10"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.15.10"
∷ word (τ ∷ ὰ ∷ ς ∷ []) "John.15.10"
∷ word (ἐ ∷ ν ∷ τ ∷ ο ∷ ∙λ ∷ ὰ ∷ ς ∷ []) "John.15.10"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.15.10"
∷ word (π ∷ α ∷ τ ∷ ρ ∷ ό ∷ ς ∷ []) "John.15.10"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.15.10"
∷ word (τ ∷ ε ∷ τ ∷ ή ∷ ρ ∷ η ∷ κ ∷ α ∷ []) "John.15.10"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.15.10"
∷ word (μ ∷ έ ∷ ν ∷ ω ∷ []) "John.15.10"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.15.10"
∷ word (ἐ ∷ ν ∷ []) "John.15.10"
∷ word (τ ∷ ῇ ∷ []) "John.15.10"
∷ word (ἀ ∷ γ ∷ ά ∷ π ∷ ῃ ∷ []) "John.15.10"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.15.11"
∷ word (∙λ ∷ ε ∷ ∙λ ∷ ά ∷ ∙λ ∷ η ∷ κ ∷ α ∷ []) "John.15.11"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.15.11"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.15.11"
∷ word (ἡ ∷ []) "John.15.11"
∷ word (χ ∷ α ∷ ρ ∷ ὰ ∷ []) "John.15.11"
∷ word (ἡ ∷ []) "John.15.11"
∷ word (ἐ ∷ μ ∷ ὴ ∷ []) "John.15.11"
∷ word (ἐ ∷ ν ∷ []) "John.15.11"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.15.11"
∷ word (ᾖ ∷ []) "John.15.11"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.15.11"
∷ word (ἡ ∷ []) "John.15.11"
∷ word (χ ∷ α ∷ ρ ∷ ὰ ∷ []) "John.15.11"
∷ word (ὑ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.15.11"
∷ word (π ∷ ∙λ ∷ η ∷ ρ ∷ ω ∷ θ ∷ ῇ ∷ []) "John.15.11"
∷ word (Α ∷ ὕ ∷ τ ∷ η ∷ []) "John.15.12"
∷ word (ἐ ∷ σ ∷ τ ∷ ὶ ∷ ν ∷ []) "John.15.12"
∷ word (ἡ ∷ []) "John.15.12"
∷ word (ἐ ∷ ν ∷ τ ∷ ο ∷ ∙λ ∷ ὴ ∷ []) "John.15.12"
∷ word (ἡ ∷ []) "John.15.12"
∷ word (ἐ ∷ μ ∷ ὴ ∷ []) "John.15.12"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.15.12"
∷ word (ἀ ∷ γ ∷ α ∷ π ∷ ᾶ ∷ τ ∷ ε ∷ []) "John.15.12"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ή ∷ ∙λ ∷ ο ∷ υ ∷ ς ∷ []) "John.15.12"
∷ word (κ ∷ α ∷ θ ∷ ὼ ∷ ς ∷ []) "John.15.12"
∷ word (ἠ ∷ γ ∷ ά ∷ π ∷ η ∷ σ ∷ α ∷ []) "John.15.12"
∷ word (ὑ ∷ μ ∷ ᾶ ∷ ς ∷ []) "John.15.12"
∷ word (μ ∷ ε ∷ ί ∷ ζ ∷ ο ∷ ν ∷ α ∷ []) "John.15.13"
∷ word (τ ∷ α ∷ ύ ∷ τ ∷ η ∷ ς ∷ []) "John.15.13"
∷ word (ἀ ∷ γ ∷ ά ∷ π ∷ η ∷ ν ∷ []) "John.15.13"
∷ word (ο ∷ ὐ ∷ δ ∷ ε ∷ ὶ ∷ ς ∷ []) "John.15.13"
∷ word (ἔ ∷ χ ∷ ε ∷ ι ∷ []) "John.15.13"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.15.13"
∷ word (τ ∷ ι ∷ ς ∷ []) "John.15.13"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.15.13"
∷ word (ψ ∷ υ ∷ χ ∷ ὴ ∷ ν ∷ []) "John.15.13"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.15.13"
∷ word (θ ∷ ῇ ∷ []) "John.15.13"
∷ word (ὑ ∷ π ∷ ὲ ∷ ρ ∷ []) "John.15.13"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.15.13"
∷ word (φ ∷ ί ∷ ∙λ ∷ ω ∷ ν ∷ []) "John.15.13"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.15.13"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.15.14"
∷ word (φ ∷ ί ∷ ∙λ ∷ ο ∷ ι ∷ []) "John.15.14"
∷ word (μ ∷ ο ∷ ύ ∷ []) "John.15.14"
∷ word (ἐ ∷ σ ∷ τ ∷ ε ∷ []) "John.15.14"
∷ word (ἐ ∷ ὰ ∷ ν ∷ []) "John.15.14"
∷ word (π ∷ ο ∷ ι ∷ ῆ ∷ τ ∷ ε ∷ []) "John.15.14"
∷ word (ἃ ∷ []) "John.15.14"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.15.14"
∷ word (ἐ ∷ ν ∷ τ ∷ έ ∷ ∙λ ∷ ∙λ ∷ ο ∷ μ ∷ α ∷ ι ∷ []) "John.15.14"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.15.14"
∷ word (ο ∷ ὐ ∷ κ ∷ έ ∷ τ ∷ ι ∷ []) "John.15.15"
∷ word (∙λ ∷ έ ∷ γ ∷ ω ∷ []) "John.15.15"
∷ word (ὑ ∷ μ ∷ ᾶ ∷ ς ∷ []) "John.15.15"
∷ word (δ ∷ ο ∷ ύ ∷ ∙λ ∷ ο ∷ υ ∷ ς ∷ []) "John.15.15"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.15.15"
∷ word (ὁ ∷ []) "John.15.15"
∷ word (δ ∷ ο ∷ ῦ ∷ ∙λ ∷ ο ∷ ς ∷ []) "John.15.15"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.15.15"
∷ word (ο ∷ ἶ ∷ δ ∷ ε ∷ ν ∷ []) "John.15.15"
∷ word (τ ∷ ί ∷ []) "John.15.15"
∷ word (π ∷ ο ∷ ι ∷ ε ∷ ῖ ∷ []) "John.15.15"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.15.15"
∷ word (ὁ ∷ []) "John.15.15"
∷ word (κ ∷ ύ ∷ ρ ∷ ι ∷ ο ∷ ς ∷ []) "John.15.15"
∷ word (ὑ ∷ μ ∷ ᾶ ∷ ς ∷ []) "John.15.15"
∷ word (δ ∷ ὲ ∷ []) "John.15.15"
∷ word (ε ∷ ἴ ∷ ρ ∷ η ∷ κ ∷ α ∷ []) "John.15.15"
∷ word (φ ∷ ί ∷ ∙λ ∷ ο ∷ υ ∷ ς ∷ []) "John.15.15"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.15.15"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ α ∷ []) "John.15.15"
∷ word (ἃ ∷ []) "John.15.15"
∷ word (ἤ ∷ κ ∷ ο ∷ υ ∷ σ ∷ α ∷ []) "John.15.15"
∷ word (π ∷ α ∷ ρ ∷ ὰ ∷ []) "John.15.15"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.15.15"
∷ word (π ∷ α ∷ τ ∷ ρ ∷ ό ∷ ς ∷ []) "John.15.15"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.15.15"
∷ word (ἐ ∷ γ ∷ ν ∷ ώ ∷ ρ ∷ ι ∷ σ ∷ α ∷ []) "John.15.15"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.15.15"
∷ word (ο ∷ ὐ ∷ χ ∷ []) "John.15.16"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.15.16"
∷ word (μ ∷ ε ∷ []) "John.15.16"
∷ word (ἐ ∷ ξ ∷ ε ∷ ∙λ ∷ έ ∷ ξ ∷ α ∷ σ ∷ θ ∷ ε ∷ []) "John.15.16"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ []) "John.15.16"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.15.16"
∷ word (ἐ ∷ ξ ∷ ε ∷ ∙λ ∷ ε ∷ ξ ∷ ά ∷ μ ∷ η ∷ ν ∷ []) "John.15.16"
∷ word (ὑ ∷ μ ∷ ᾶ ∷ ς ∷ []) "John.15.16"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.15.16"
∷ word (ἔ ∷ θ ∷ η ∷ κ ∷ α ∷ []) "John.15.16"
∷ word (ὑ ∷ μ ∷ ᾶ ∷ ς ∷ []) "John.15.16"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.15.16"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.15.16"
∷ word (ὑ ∷ π ∷ ά ∷ γ ∷ η ∷ τ ∷ ε ∷ []) "John.15.16"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.15.16"
∷ word (κ ∷ α ∷ ρ ∷ π ∷ ὸ ∷ ν ∷ []) "John.15.16"
∷ word (φ ∷ έ ∷ ρ ∷ η ∷ τ ∷ ε ∷ []) "John.15.16"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.15.16"
∷ word (ὁ ∷ []) "John.15.16"
∷ word (κ ∷ α ∷ ρ ∷ π ∷ ὸ ∷ ς ∷ []) "John.15.16"
∷ word (ὑ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.15.16"
∷ word (μ ∷ έ ∷ ν ∷ ῃ ∷ []) "John.15.16"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.15.16"
∷ word (ὅ ∷ []) "John.15.16"
∷ word (τ ∷ ι ∷ []) "John.15.16"
∷ word (ἂ ∷ ν ∷ []) "John.15.16"
∷ word (α ∷ ἰ ∷ τ ∷ ή ∷ σ ∷ η ∷ τ ∷ ε ∷ []) "John.15.16"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.15.16"
∷ word (π ∷ α ∷ τ ∷ έ ∷ ρ ∷ α ∷ []) "John.15.16"
∷ word (ἐ ∷ ν ∷ []) "John.15.16"
∷ word (τ ∷ ῷ ∷ []) "John.15.16"
∷ word (ὀ ∷ ν ∷ ό ∷ μ ∷ α ∷ τ ∷ ί ∷ []) "John.15.16"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.15.16"
∷ word (δ ∷ ῷ ∷ []) "John.15.16"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.15.16"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.15.17"
∷ word (ἐ ∷ ν ∷ τ ∷ έ ∷ ∙λ ∷ ∙λ ∷ ο ∷ μ ∷ α ∷ ι ∷ []) "John.15.17"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.15.17"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.15.17"
∷ word (ἀ ∷ γ ∷ α ∷ π ∷ ᾶ ∷ τ ∷ ε ∷ []) "John.15.17"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ή ∷ ∙λ ∷ ο ∷ υ ∷ ς ∷ []) "John.15.17"
∷ word (Ε ∷ ἰ ∷ []) "John.15.18"
∷ word (ὁ ∷ []) "John.15.18"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ ς ∷ []) "John.15.18"
∷ word (ὑ ∷ μ ∷ ᾶ ∷ ς ∷ []) "John.15.18"
∷ word (μ ∷ ι ∷ σ ∷ ε ∷ ῖ ∷ []) "John.15.18"
∷ word (γ ∷ ι ∷ ν ∷ ώ ∷ σ ∷ κ ∷ ε ∷ τ ∷ ε ∷ []) "John.15.18"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.15.18"
∷ word (ἐ ∷ μ ∷ ὲ ∷ []) "John.15.18"
∷ word (π ∷ ρ ∷ ῶ ∷ τ ∷ ο ∷ ν ∷ []) "John.15.18"
∷ word (ὑ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.15.18"
∷ word (μ ∷ ε ∷ μ ∷ ί ∷ σ ∷ η ∷ κ ∷ ε ∷ ν ∷ []) "John.15.18"
∷ word (ε ∷ ἰ ∷ []) "John.15.19"
∷ word (ἐ ∷ κ ∷ []) "John.15.19"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.15.19"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ υ ∷ []) "John.15.19"
∷ word (ἦ ∷ τ ∷ ε ∷ []) "John.15.19"
∷ word (ὁ ∷ []) "John.15.19"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ ς ∷ []) "John.15.19"
∷ word (ἂ ∷ ν ∷ []) "John.15.19"
∷ word (τ ∷ ὸ ∷ []) "John.15.19"
∷ word (ἴ ∷ δ ∷ ι ∷ ο ∷ ν ∷ []) "John.15.19"
∷ word (ἐ ∷ φ ∷ ί ∷ ∙λ ∷ ε ∷ ι ∷ []) "John.15.19"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.15.19"
∷ word (δ ∷ ὲ ∷ []) "John.15.19"
∷ word (ἐ ∷ κ ∷ []) "John.15.19"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.15.19"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ υ ∷ []) "John.15.19"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.15.19"
∷ word (ἐ ∷ σ ∷ τ ∷ έ ∷ []) "John.15.19"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ []) "John.15.19"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.15.19"
∷ word (ἐ ∷ ξ ∷ ε ∷ ∙λ ∷ ε ∷ ξ ∷ ά ∷ μ ∷ η ∷ ν ∷ []) "John.15.19"
∷ word (ὑ ∷ μ ∷ ᾶ ∷ ς ∷ []) "John.15.19"
∷ word (ἐ ∷ κ ∷ []) "John.15.19"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.15.19"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ υ ∷ []) "John.15.19"
∷ word (δ ∷ ι ∷ ὰ ∷ []) "John.15.19"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.15.19"
∷ word (μ ∷ ι ∷ σ ∷ ε ∷ ῖ ∷ []) "John.15.19"
∷ word (ὑ ∷ μ ∷ ᾶ ∷ ς ∷ []) "John.15.19"
∷ word (ὁ ∷ []) "John.15.19"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ ς ∷ []) "John.15.19"
∷ word (μ ∷ ν ∷ η ∷ μ ∷ ο ∷ ν ∷ ε ∷ ύ ∷ ε ∷ τ ∷ ε ∷ []) "John.15.20"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.15.20"
∷ word (∙λ ∷ ό ∷ γ ∷ ο ∷ υ ∷ []) "John.15.20"
∷ word (ο ∷ ὗ ∷ []) "John.15.20"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.15.20"
∷ word (ε ∷ ἶ ∷ π ∷ ο ∷ ν ∷ []) "John.15.20"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.15.20"
∷ word (Ο ∷ ὐ ∷ κ ∷ []) "John.15.20"
∷ word (ἔ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.15.20"
∷ word (δ ∷ ο ∷ ῦ ∷ ∙λ ∷ ο ∷ ς ∷ []) "John.15.20"
∷ word (μ ∷ ε ∷ ί ∷ ζ ∷ ω ∷ ν ∷ []) "John.15.20"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.15.20"
∷ word (κ ∷ υ ∷ ρ ∷ ί ∷ ο ∷ υ ∷ []) "John.15.20"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.15.20"
∷ word (ε ∷ ἰ ∷ []) "John.15.20"
∷ word (ἐ ∷ μ ∷ ὲ ∷ []) "John.15.20"
∷ word (ἐ ∷ δ ∷ ί ∷ ω ∷ ξ ∷ α ∷ ν ∷ []) "John.15.20"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.15.20"
∷ word (ὑ ∷ μ ∷ ᾶ ∷ ς ∷ []) "John.15.20"
∷ word (δ ∷ ι ∷ ώ ∷ ξ ∷ ο ∷ υ ∷ σ ∷ ι ∷ ν ∷ []) "John.15.20"
∷ word (ε ∷ ἰ ∷ []) "John.15.20"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.15.20"
∷ word (∙λ ∷ ό ∷ γ ∷ ο ∷ ν ∷ []) "John.15.20"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.15.20"
∷ word (ἐ ∷ τ ∷ ή ∷ ρ ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.15.20"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.15.20"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.15.20"
∷ word (ὑ ∷ μ ∷ έ ∷ τ ∷ ε ∷ ρ ∷ ο ∷ ν ∷ []) "John.15.20"
∷ word (τ ∷ η ∷ ρ ∷ ή ∷ σ ∷ ο ∷ υ ∷ σ ∷ ι ∷ ν ∷ []) "John.15.20"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.15.21"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.15.21"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ α ∷ []) "John.15.21"
∷ word (π ∷ ο ∷ ι ∷ ή ∷ σ ∷ ο ∷ υ ∷ σ ∷ ι ∷ ν ∷ []) "John.15.21"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.15.21"
∷ word (ὑ ∷ μ ∷ ᾶ ∷ ς ∷ []) "John.15.21"
∷ word (δ ∷ ι ∷ ὰ ∷ []) "John.15.21"
∷ word (τ ∷ ὸ ∷ []) "John.15.21"
∷ word (ὄ ∷ ν ∷ ο ∷ μ ∷ ά ∷ []) "John.15.21"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.15.21"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.15.21"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.15.21"
∷ word (ο ∷ ἴ ∷ δ ∷ α ∷ σ ∷ ι ∷ ν ∷ []) "John.15.21"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.15.21"
∷ word (π ∷ έ ∷ μ ∷ ψ ∷ α ∷ ν ∷ τ ∷ ά ∷ []) "John.15.21"
∷ word (μ ∷ ε ∷ []) "John.15.21"
∷ word (ε ∷ ἰ ∷ []) "John.15.22"
∷ word (μ ∷ ὴ ∷ []) "John.15.22"
∷ word (ἦ ∷ ∙λ ∷ θ ∷ ο ∷ ν ∷ []) "John.15.22"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.15.22"
∷ word (ἐ ∷ ∙λ ∷ ά ∷ ∙λ ∷ η ∷ σ ∷ α ∷ []) "John.15.22"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.15.22"
∷ word (ἁ ∷ μ ∷ α ∷ ρ ∷ τ ∷ ί ∷ α ∷ ν ∷ []) "John.15.22"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.15.22"
∷ word (ε ∷ ἴ ∷ χ ∷ ο ∷ σ ∷ α ∷ ν ∷ []) "John.15.22"
∷ word (ν ∷ ῦ ∷ ν ∷ []) "John.15.22"
∷ word (δ ∷ ὲ ∷ []) "John.15.22"
∷ word (π ∷ ρ ∷ ό ∷ φ ∷ α ∷ σ ∷ ι ∷ ν ∷ []) "John.15.22"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.15.22"
∷ word (ἔ ∷ χ ∷ ο ∷ υ ∷ σ ∷ ι ∷ ν ∷ []) "John.15.22"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.15.22"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.15.22"
∷ word (ἁ ∷ μ ∷ α ∷ ρ ∷ τ ∷ ί ∷ α ∷ ς ∷ []) "John.15.22"
∷ word (α ∷ ὐ ∷ τ ∷ ῶ ∷ ν ∷ []) "John.15.22"
∷ word (ὁ ∷ []) "John.15.23"
∷ word (ἐ ∷ μ ∷ ὲ ∷ []) "John.15.23"
∷ word (μ ∷ ι ∷ σ ∷ ῶ ∷ ν ∷ []) "John.15.23"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.15.23"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.15.23"
∷ word (π ∷ α ∷ τ ∷ έ ∷ ρ ∷ α ∷ []) "John.15.23"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.15.23"
∷ word (μ ∷ ι ∷ σ ∷ ε ∷ ῖ ∷ []) "John.15.23"
∷ word (ε ∷ ἰ ∷ []) "John.15.24"
∷ word (τ ∷ ὰ ∷ []) "John.15.24"
∷ word (ἔ ∷ ρ ∷ γ ∷ α ∷ []) "John.15.24"
∷ word (μ ∷ ὴ ∷ []) "John.15.24"
∷ word (ἐ ∷ π ∷ ο ∷ ί ∷ η ∷ σ ∷ α ∷ []) "John.15.24"
∷ word (ἐ ∷ ν ∷ []) "John.15.24"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.15.24"
∷ word (ἃ ∷ []) "John.15.24"
∷ word (ο ∷ ὐ ∷ δ ∷ ε ∷ ὶ ∷ ς ∷ []) "John.15.24"
∷ word (ἄ ∷ ∙λ ∷ ∙λ ∷ ο ∷ ς ∷ []) "John.15.24"
∷ word (ἐ ∷ π ∷ ο ∷ ί ∷ η ∷ σ ∷ ε ∷ ν ∷ []) "John.15.24"
∷ word (ἁ ∷ μ ∷ α ∷ ρ ∷ τ ∷ ί ∷ α ∷ ν ∷ []) "John.15.24"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.15.24"
∷ word (ε ∷ ἴ ∷ χ ∷ ο ∷ σ ∷ α ∷ ν ∷ []) "John.15.24"
∷ word (ν ∷ ῦ ∷ ν ∷ []) "John.15.24"
∷ word (δ ∷ ὲ ∷ []) "John.15.24"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.15.24"
∷ word (ἑ ∷ ω ∷ ρ ∷ ά ∷ κ ∷ α ∷ σ ∷ ι ∷ ν ∷ []) "John.15.24"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.15.24"
∷ word (μ ∷ ε ∷ μ ∷ ι ∷ σ ∷ ή ∷ κ ∷ α ∷ σ ∷ ι ∷ ν ∷ []) "John.15.24"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.15.24"
∷ word (ἐ ∷ μ ∷ ὲ ∷ []) "John.15.24"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.15.24"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.15.24"
∷ word (π ∷ α ∷ τ ∷ έ ∷ ρ ∷ α ∷ []) "John.15.24"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.15.24"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ []) "John.15.25"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.15.25"
∷ word (π ∷ ∙λ ∷ η ∷ ρ ∷ ω ∷ θ ∷ ῇ ∷ []) "John.15.25"
∷ word (ὁ ∷ []) "John.15.25"
∷ word (∙λ ∷ ό ∷ γ ∷ ο ∷ ς ∷ []) "John.15.25"
∷ word (ὁ ∷ []) "John.15.25"
∷ word (ἐ ∷ ν ∷ []) "John.15.25"
∷ word (τ ∷ ῷ ∷ []) "John.15.25"
∷ word (ν ∷ ό ∷ μ ∷ ῳ ∷ []) "John.15.25"
∷ word (α ∷ ὐ ∷ τ ∷ ῶ ∷ ν ∷ []) "John.15.25"
∷ word (γ ∷ ε ∷ γ ∷ ρ ∷ α ∷ μ ∷ μ ∷ έ ∷ ν ∷ ο ∷ ς ∷ []) "John.15.25"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.15.25"
∷ word (Ἐ ∷ μ ∷ ί ∷ σ ∷ η ∷ σ ∷ ά ∷ ν ∷ []) "John.15.25"
∷ word (μ ∷ ε ∷ []) "John.15.25"
∷ word (δ ∷ ω ∷ ρ ∷ ε ∷ ά ∷ ν ∷ []) "John.15.25"
∷ word (Ὅ ∷ τ ∷ α ∷ ν ∷ []) "John.15.26"
∷ word (ἔ ∷ ∙λ ∷ θ ∷ ῃ ∷ []) "John.15.26"
∷ word (ὁ ∷ []) "John.15.26"
∷ word (π ∷ α ∷ ρ ∷ ά ∷ κ ∷ ∙λ ∷ η ∷ τ ∷ ο ∷ ς ∷ []) "John.15.26"
∷ word (ὃ ∷ ν ∷ []) "John.15.26"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.15.26"
∷ word (π ∷ έ ∷ μ ∷ ψ ∷ ω ∷ []) "John.15.26"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.15.26"
∷ word (π ∷ α ∷ ρ ∷ ὰ ∷ []) "John.15.26"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.15.26"
∷ word (π ∷ α ∷ τ ∷ ρ ∷ ό ∷ ς ∷ []) "John.15.26"
∷ word (τ ∷ ὸ ∷ []) "John.15.26"
∷ word (π ∷ ν ∷ ε ∷ ῦ ∷ μ ∷ α ∷ []) "John.15.26"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.15.26"
∷ word (ἀ ∷ ∙λ ∷ η ∷ θ ∷ ε ∷ ί ∷ α ∷ ς ∷ []) "John.15.26"
∷ word (ὃ ∷ []) "John.15.26"
∷ word (π ∷ α ∷ ρ ∷ ὰ ∷ []) "John.15.26"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.15.26"
∷ word (π ∷ α ∷ τ ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.15.26"
∷ word (ἐ ∷ κ ∷ π ∷ ο ∷ ρ ∷ ε ∷ ύ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.15.26"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ο ∷ ς ∷ []) "John.15.26"
∷ word (μ ∷ α ∷ ρ ∷ τ ∷ υ ∷ ρ ∷ ή ∷ σ ∷ ε ∷ ι ∷ []) "John.15.26"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.15.26"
∷ word (ἐ ∷ μ ∷ ο ∷ ῦ ∷ []) "John.15.26"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.15.27"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.15.27"
∷ word (δ ∷ ὲ ∷ []) "John.15.27"
∷ word (μ ∷ α ∷ ρ ∷ τ ∷ υ ∷ ρ ∷ ε ∷ ῖ ∷ τ ∷ ε ∷ []) "John.15.27"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.15.27"
∷ word (ἀ ∷ π ∷ []) "John.15.27"
∷ word (ἀ ∷ ρ ∷ χ ∷ ῆ ∷ ς ∷ []) "John.15.27"
∷ word (μ ∷ ε ∷ τ ∷ []) "John.15.27"
∷ word (ἐ ∷ μ ∷ ο ∷ ῦ ∷ []) "John.15.27"
∷ word (ἐ ∷ σ ∷ τ ∷ ε ∷ []) "John.15.27"
∷ word (Τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.16.1"
∷ word (∙λ ∷ ε ∷ ∙λ ∷ ά ∷ ∙λ ∷ η ∷ κ ∷ α ∷ []) "John.16.1"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.16.1"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.16.1"
∷ word (μ ∷ ὴ ∷ []) "John.16.1"
∷ word (σ ∷ κ ∷ α ∷ ν ∷ δ ∷ α ∷ ∙λ ∷ ι ∷ σ ∷ θ ∷ ῆ ∷ τ ∷ ε ∷ []) "John.16.1"
∷ word (ἀ ∷ π ∷ ο ∷ σ ∷ υ ∷ ν ∷ α ∷ γ ∷ ώ ∷ γ ∷ ο ∷ υ ∷ ς ∷ []) "John.16.2"
∷ word (π ∷ ο ∷ ι ∷ ή ∷ σ ∷ ο ∷ υ ∷ σ ∷ ι ∷ ν ∷ []) "John.16.2"
∷ word (ὑ ∷ μ ∷ ᾶ ∷ ς ∷ []) "John.16.2"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ []) "John.16.2"
∷ word (ἔ ∷ ρ ∷ χ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.16.2"
∷ word (ὥ ∷ ρ ∷ α ∷ []) "John.16.2"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.16.2"
∷ word (π ∷ ᾶ ∷ ς ∷ []) "John.16.2"
∷ word (ὁ ∷ []) "John.16.2"
∷ word (ἀ ∷ π ∷ ο ∷ κ ∷ τ ∷ ε ∷ ί ∷ ν ∷ α ∷ ς ∷ []) "John.16.2"
∷ word (ὑ ∷ μ ∷ ᾶ ∷ ς ∷ []) "John.16.2"
∷ word (δ ∷ ό ∷ ξ ∷ ῃ ∷ []) "John.16.2"
∷ word (∙λ ∷ α ∷ τ ∷ ρ ∷ ε ∷ ί ∷ α ∷ ν ∷ []) "John.16.2"
∷ word (π ∷ ρ ∷ ο ∷ σ ∷ φ ∷ έ ∷ ρ ∷ ε ∷ ι ∷ ν ∷ []) "John.16.2"
∷ word (τ ∷ ῷ ∷ []) "John.16.2"
∷ word (θ ∷ ε ∷ ῷ ∷ []) "John.16.2"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.16.3"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.16.3"
∷ word (π ∷ ο ∷ ι ∷ ή ∷ σ ∷ ο ∷ υ ∷ σ ∷ ι ∷ ν ∷ []) "John.16.3"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.16.3"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.16.3"
∷ word (ἔ ∷ γ ∷ ν ∷ ω ∷ σ ∷ α ∷ ν ∷ []) "John.16.3"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.16.3"
∷ word (π ∷ α ∷ τ ∷ έ ∷ ρ ∷ α ∷ []) "John.16.3"
∷ word (ο ∷ ὐ ∷ δ ∷ ὲ ∷ []) "John.16.3"
∷ word (ἐ ∷ μ ∷ έ ∷ []) "John.16.3"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.16.4"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.16.4"
∷ word (∙λ ∷ ε ∷ ∙λ ∷ ά ∷ ∙λ ∷ η ∷ κ ∷ α ∷ []) "John.16.4"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.16.4"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.16.4"
∷ word (ὅ ∷ τ ∷ α ∷ ν ∷ []) "John.16.4"
∷ word (ἔ ∷ ∙λ ∷ θ ∷ ῃ ∷ []) "John.16.4"
∷ word (ἡ ∷ []) "John.16.4"
∷ word (ὥ ∷ ρ ∷ α ∷ []) "John.16.4"
∷ word (α ∷ ὐ ∷ τ ∷ ῶ ∷ ν ∷ []) "John.16.4"
∷ word (μ ∷ ν ∷ η ∷ μ ∷ ο ∷ ν ∷ ε ∷ ύ ∷ η ∷ τ ∷ ε ∷ []) "John.16.4"
∷ word (α ∷ ὐ ∷ τ ∷ ῶ ∷ ν ∷ []) "John.16.4"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.16.4"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.16.4"
∷ word (ε ∷ ἶ ∷ π ∷ ο ∷ ν ∷ []) "John.16.4"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.16.4"
∷ word (Τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.16.4"
∷ word (δ ∷ ὲ ∷ []) "John.16.4"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.16.4"
∷ word (ἐ ∷ ξ ∷ []) "John.16.4"
∷ word (ἀ ∷ ρ ∷ χ ∷ ῆ ∷ ς ∷ []) "John.16.4"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.16.4"
∷ word (ε ∷ ἶ ∷ π ∷ ο ∷ ν ∷ []) "John.16.4"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.16.4"
∷ word (μ ∷ ε ∷ θ ∷ []) "John.16.4"
∷ word (ὑ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.16.4"
∷ word (ἤ ∷ μ ∷ η ∷ ν ∷ []) "John.16.4"
∷ word (ν ∷ ῦ ∷ ν ∷ []) "John.16.5"
∷ word (δ ∷ ὲ ∷ []) "John.16.5"
∷ word (ὑ ∷ π ∷ ά ∷ γ ∷ ω ∷ []) "John.16.5"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.16.5"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.16.5"
∷ word (π ∷ έ ∷ μ ∷ ψ ∷ α ∷ ν ∷ τ ∷ ά ∷ []) "John.16.5"
∷ word (μ ∷ ε ∷ []) "John.16.5"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.16.5"
∷ word (ο ∷ ὐ ∷ δ ∷ ε ∷ ὶ ∷ ς ∷ []) "John.16.5"
∷ word (ἐ ∷ ξ ∷ []) "John.16.5"
∷ word (ὑ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.16.5"
∷ word (ἐ ∷ ρ ∷ ω ∷ τ ∷ ᾷ ∷ []) "John.16.5"
∷ word (μ ∷ ε ∷ []) "John.16.5"
∷ word (Π ∷ ο ∷ ῦ ∷ []) "John.16.5"
∷ word (ὑ ∷ π ∷ ά ∷ γ ∷ ε ∷ ι ∷ ς ∷ []) "John.16.5"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ []) "John.16.6"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.16.6"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.16.6"
∷ word (∙λ ∷ ε ∷ ∙λ ∷ ά ∷ ∙λ ∷ η ∷ κ ∷ α ∷ []) "John.16.6"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.16.6"
∷ word (ἡ ∷ []) "John.16.6"
∷ word (∙λ ∷ ύ ∷ π ∷ η ∷ []) "John.16.6"
∷ word (π ∷ ε ∷ π ∷ ∙λ ∷ ή ∷ ρ ∷ ω ∷ κ ∷ ε ∷ ν ∷ []) "John.16.6"
∷ word (ὑ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.16.6"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.16.6"
∷ word (κ ∷ α ∷ ρ ∷ δ ∷ ί ∷ α ∷ ν ∷ []) "John.16.6"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ []) "John.16.7"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.16.7"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.16.7"
∷ word (ἀ ∷ ∙λ ∷ ή ∷ θ ∷ ε ∷ ι ∷ α ∷ ν ∷ []) "John.16.7"
∷ word (∙λ ∷ έ ∷ γ ∷ ω ∷ []) "John.16.7"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.16.7"
∷ word (σ ∷ υ ∷ μ ∷ φ ∷ έ ∷ ρ ∷ ε ∷ ι ∷ []) "John.16.7"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.16.7"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.16.7"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.16.7"
∷ word (ἀ ∷ π ∷ έ ∷ ∙λ ∷ θ ∷ ω ∷ []) "John.16.7"
∷ word (ἐ ∷ ὰ ∷ ν ∷ []) "John.16.7"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.16.7"
∷ word (μ ∷ ὴ ∷ []) "John.16.7"
∷ word (ἀ ∷ π ∷ έ ∷ ∙λ ∷ θ ∷ ω ∷ []) "John.16.7"
∷ word (ὁ ∷ []) "John.16.7"
∷ word (π ∷ α ∷ ρ ∷ ά ∷ κ ∷ ∙λ ∷ η ∷ τ ∷ ο ∷ ς ∷ []) "John.16.7"
∷ word (ο ∷ ὐ ∷ []) "John.16.7"
∷ word (μ ∷ ὴ ∷ []) "John.16.7"
∷ word (ἔ ∷ ∙λ ∷ θ ∷ ῃ ∷ []) "John.16.7"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.16.7"
∷ word (ὑ ∷ μ ∷ ᾶ ∷ ς ∷ []) "John.16.7"
∷ word (ἐ ∷ ὰ ∷ ν ∷ []) "John.16.7"
∷ word (δ ∷ ὲ ∷ []) "John.16.7"
∷ word (π ∷ ο ∷ ρ ∷ ε ∷ υ ∷ θ ∷ ῶ ∷ []) "John.16.7"
∷ word (π ∷ έ ∷ μ ∷ ψ ∷ ω ∷ []) "John.16.7"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.16.7"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.16.7"
∷ word (ὑ ∷ μ ∷ ᾶ ∷ ς ∷ []) "John.16.7"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.16.8"
∷ word (ἐ ∷ ∙λ ∷ θ ∷ ὼ ∷ ν ∷ []) "John.16.8"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ο ∷ ς ∷ []) "John.16.8"
∷ word (ἐ ∷ ∙λ ∷ έ ∷ γ ∷ ξ ∷ ε ∷ ι ∷ []) "John.16.8"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.16.8"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ ν ∷ []) "John.16.8"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.16.8"
∷ word (ἁ ∷ μ ∷ α ∷ ρ ∷ τ ∷ ί ∷ α ∷ ς ∷ []) "John.16.8"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.16.8"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.16.8"
∷ word (δ ∷ ι ∷ κ ∷ α ∷ ι ∷ ο ∷ σ ∷ ύ ∷ ν ∷ η ∷ ς ∷ []) "John.16.8"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.16.8"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.16.8"
∷ word (κ ∷ ρ ∷ ί ∷ σ ∷ ε ∷ ω ∷ ς ∷ []) "John.16.8"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.16.9"
∷ word (ἁ ∷ μ ∷ α ∷ ρ ∷ τ ∷ ί ∷ α ∷ ς ∷ []) "John.16.9"
∷ word (μ ∷ έ ∷ ν ∷ []) "John.16.9"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.16.9"
∷ word (ο ∷ ὐ ∷ []) "John.16.9"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ ο ∷ υ ∷ σ ∷ ι ∷ ν ∷ []) "John.16.9"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.16.9"
∷ word (ἐ ∷ μ ∷ έ ∷ []) "John.16.9"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.16.10"
∷ word (δ ∷ ι ∷ κ ∷ α ∷ ι ∷ ο ∷ σ ∷ ύ ∷ ν ∷ η ∷ ς ∷ []) "John.16.10"
∷ word (δ ∷ έ ∷ []) "John.16.10"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.16.10"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.16.10"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.16.10"
∷ word (π ∷ α ∷ τ ∷ έ ∷ ρ ∷ α ∷ []) "John.16.10"
∷ word (ὑ ∷ π ∷ ά ∷ γ ∷ ω ∷ []) "John.16.10"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.16.10"
∷ word (ο ∷ ὐ ∷ κ ∷ έ ∷ τ ∷ ι ∷ []) "John.16.10"
∷ word (θ ∷ ε ∷ ω ∷ ρ ∷ ε ∷ ῖ ∷ τ ∷ έ ∷ []) "John.16.10"
∷ word (μ ∷ ε ∷ []) "John.16.10"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.16.11"
∷ word (δ ∷ ὲ ∷ []) "John.16.11"
∷ word (κ ∷ ρ ∷ ί ∷ σ ∷ ε ∷ ω ∷ ς ∷ []) "John.16.11"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.16.11"
∷ word (ὁ ∷ []) "John.16.11"
∷ word (ἄ ∷ ρ ∷ χ ∷ ω ∷ ν ∷ []) "John.16.11"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.16.11"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ υ ∷ []) "John.16.11"
∷ word (τ ∷ ο ∷ ύ ∷ τ ∷ ο ∷ υ ∷ []) "John.16.11"
∷ word (κ ∷ έ ∷ κ ∷ ρ ∷ ι ∷ τ ∷ α ∷ ι ∷ []) "John.16.11"
∷ word (Ἔ ∷ τ ∷ ι ∷ []) "John.16.12"
∷ word (π ∷ ο ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.16.12"
∷ word (ἔ ∷ χ ∷ ω ∷ []) "John.16.12"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.16.12"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ ν ∷ []) "John.16.12"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ []) "John.16.12"
∷ word (ο ∷ ὐ ∷ []) "John.16.12"
∷ word (δ ∷ ύ ∷ ν ∷ α ∷ σ ∷ θ ∷ ε ∷ []) "John.16.12"
∷ word (β ∷ α ∷ σ ∷ τ ∷ ά ∷ ζ ∷ ε ∷ ι ∷ ν ∷ []) "John.16.12"
∷ word (ἄ ∷ ρ ∷ τ ∷ ι ∷ []) "John.16.12"
∷ word (ὅ ∷ τ ∷ α ∷ ν ∷ []) "John.16.13"
∷ word (δ ∷ ὲ ∷ []) "John.16.13"
∷ word (ἔ ∷ ∙λ ∷ θ ∷ ῃ ∷ []) "John.16.13"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ο ∷ ς ∷ []) "John.16.13"
∷ word (τ ∷ ὸ ∷ []) "John.16.13"
∷ word (π ∷ ν ∷ ε ∷ ῦ ∷ μ ∷ α ∷ []) "John.16.13"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.16.13"
∷ word (ἀ ∷ ∙λ ∷ η ∷ θ ∷ ε ∷ ί ∷ α ∷ ς ∷ []) "John.16.13"
∷ word (ὁ ∷ δ ∷ η ∷ γ ∷ ή ∷ σ ∷ ε ∷ ι ∷ []) "John.16.13"
∷ word (ὑ ∷ μ ∷ ᾶ ∷ ς ∷ []) "John.16.13"
∷ word (ἐ ∷ ν ∷ []) "John.16.13"
∷ word (τ ∷ ῇ ∷ []) "John.16.13"
∷ word (ἀ ∷ ∙λ ∷ η ∷ θ ∷ ε ∷ ί ∷ ᾳ ∷ []) "John.16.13"
∷ word (π ∷ ά ∷ σ ∷ ῃ ∷ []) "John.16.13"
∷ word (ο ∷ ὐ ∷ []) "John.16.13"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.16.13"
∷ word (∙λ ∷ α ∷ ∙λ ∷ ή ∷ σ ∷ ε ∷ ι ∷ []) "John.16.13"
∷ word (ἀ ∷ φ ∷ []) "John.16.13"
∷ word (ἑ ∷ α ∷ υ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.16.13"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ []) "John.16.13"
∷ word (ὅ ∷ σ ∷ α ∷ []) "John.16.13"
∷ word (ἀ ∷ κ ∷ ο ∷ ύ ∷ σ ∷ ε ∷ ι ∷ []) "John.16.13"
∷ word (∙λ ∷ α ∷ ∙λ ∷ ή ∷ σ ∷ ε ∷ ι ∷ []) "John.16.13"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.16.13"
∷ word (τ ∷ ὰ ∷ []) "John.16.13"
∷ word (ἐ ∷ ρ ∷ χ ∷ ό ∷ μ ∷ ε ∷ ν ∷ α ∷ []) "John.16.13"
∷ word (ἀ ∷ ν ∷ α ∷ γ ∷ γ ∷ ε ∷ ∙λ ∷ ε ∷ ῖ ∷ []) "John.16.13"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.16.13"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ο ∷ ς ∷ []) "John.16.14"
∷ word (ἐ ∷ μ ∷ ὲ ∷ []) "John.16.14"
∷ word (δ ∷ ο ∷ ξ ∷ ά ∷ σ ∷ ε ∷ ι ∷ []) "John.16.14"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.16.14"
∷ word (ἐ ∷ κ ∷ []) "John.16.14"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.16.14"
∷ word (ἐ ∷ μ ∷ ο ∷ ῦ ∷ []) "John.16.14"
∷ word (∙λ ∷ ή ∷ μ ∷ ψ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.16.14"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.16.14"
∷ word (ἀ ∷ ν ∷ α ∷ γ ∷ γ ∷ ε ∷ ∙λ ∷ ε ∷ ῖ ∷ []) "John.16.14"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.16.14"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ α ∷ []) "John.16.15"
∷ word (ὅ ∷ σ ∷ α ∷ []) "John.16.15"
∷ word (ἔ ∷ χ ∷ ε ∷ ι ∷ []) "John.16.15"
∷ word (ὁ ∷ []) "John.16.15"
∷ word (π ∷ α ∷ τ ∷ ὴ ∷ ρ ∷ []) "John.16.15"
∷ word (ἐ ∷ μ ∷ ά ∷ []) "John.16.15"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.16.15"
∷ word (δ ∷ ι ∷ ὰ ∷ []) "John.16.15"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.16.15"
∷ word (ε ∷ ἶ ∷ π ∷ ο ∷ ν ∷ []) "John.16.15"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.16.15"
∷ word (ἐ ∷ κ ∷ []) "John.16.15"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.16.15"
∷ word (ἐ ∷ μ ∷ ο ∷ ῦ ∷ []) "John.16.15"
∷ word (∙λ ∷ α ∷ μ ∷ β ∷ ά ∷ ν ∷ ε ∷ ι ∷ []) "John.16.15"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.16.15"
∷ word (ἀ ∷ ν ∷ α ∷ γ ∷ γ ∷ ε ∷ ∙λ ∷ ε ∷ ῖ ∷ []) "John.16.15"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.16.15"
∷ word (Μ ∷ ι ∷ κ ∷ ρ ∷ ὸ ∷ ν ∷ []) "John.16.16"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.16.16"
∷ word (ο ∷ ὐ ∷ κ ∷ έ ∷ τ ∷ ι ∷ []) "John.16.16"
∷ word (θ ∷ ε ∷ ω ∷ ρ ∷ ε ∷ ῖ ∷ τ ∷ έ ∷ []) "John.16.16"
∷ word (μ ∷ ε ∷ []) "John.16.16"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.16.16"
∷ word (π ∷ ά ∷ ∙λ ∷ ι ∷ ν ∷ []) "John.16.16"
∷ word (μ ∷ ι ∷ κ ∷ ρ ∷ ὸ ∷ ν ∷ []) "John.16.16"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.16.16"
∷ word (ὄ ∷ ψ ∷ ε ∷ σ ∷ θ ∷ έ ∷ []) "John.16.16"
∷ word (μ ∷ ε ∷ []) "John.16.16"
∷ word (ε ∷ ἶ ∷ π ∷ α ∷ ν ∷ []) "John.16.17"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.16.17"
∷ word (ἐ ∷ κ ∷ []) "John.16.17"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.16.17"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ ῶ ∷ ν ∷ []) "John.16.17"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.16.17"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.16.17"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ή ∷ ∙λ ∷ ο ∷ υ ∷ ς ∷ []) "John.16.17"
∷ word (Τ ∷ ί ∷ []) "John.16.17"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.16.17"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.16.17"
∷ word (ὃ ∷ []) "John.16.17"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.16.17"
∷ word (ἡ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.16.17"
∷ word (Μ ∷ ι ∷ κ ∷ ρ ∷ ὸ ∷ ν ∷ []) "John.16.17"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.16.17"
∷ word (ο ∷ ὐ ∷ []) "John.16.17"
∷ word (θ ∷ ε ∷ ω ∷ ρ ∷ ε ∷ ῖ ∷ τ ∷ έ ∷ []) "John.16.17"
∷ word (μ ∷ ε ∷ []) "John.16.17"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.16.17"
∷ word (π ∷ ά ∷ ∙λ ∷ ι ∷ ν ∷ []) "John.16.17"
∷ word (μ ∷ ι ∷ κ ∷ ρ ∷ ὸ ∷ ν ∷ []) "John.16.17"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.16.17"
∷ word (ὄ ∷ ψ ∷ ε ∷ σ ∷ θ ∷ έ ∷ []) "John.16.17"
∷ word (μ ∷ ε ∷ []) "John.16.17"
∷ word (κ ∷ α ∷ ί ∷ []) "John.16.17"
∷ word (Ὅ ∷ τ ∷ ι ∷ []) "John.16.17"
∷ word (ὑ ∷ π ∷ ά ∷ γ ∷ ω ∷ []) "John.16.17"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.16.17"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.16.17"
∷ word (π ∷ α ∷ τ ∷ έ ∷ ρ ∷ α ∷ []) "John.16.17"
∷ word (ἔ ∷ ∙λ ∷ ε ∷ γ ∷ ο ∷ ν ∷ []) "John.16.18"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.16.18"
∷ word (Τ ∷ ί ∷ []) "John.16.18"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.16.18"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.16.18"
∷ word (ὃ ∷ []) "John.16.18"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.16.18"
∷ word (μ ∷ ι ∷ κ ∷ ρ ∷ ό ∷ ν ∷ []) "John.16.18"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.16.18"
∷ word (ο ∷ ἴ ∷ δ ∷ α ∷ μ ∷ ε ∷ ν ∷ []) "John.16.18"
∷ word (τ ∷ ί ∷ []) "John.16.18"
∷ word (∙λ ∷ α ∷ ∙λ ∷ ε ∷ ῖ ∷ []) "John.16.18"
∷ word (ἔ ∷ γ ∷ ν ∷ ω ∷ []) "John.16.19"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.16.19"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.16.19"
∷ word (ἤ ∷ θ ∷ ε ∷ ∙λ ∷ ο ∷ ν ∷ []) "John.16.19"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.16.19"
∷ word (ἐ ∷ ρ ∷ ω ∷ τ ∷ ᾶ ∷ ν ∷ []) "John.16.19"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.16.19"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.16.19"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.16.19"
∷ word (Π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.16.19"
∷ word (τ ∷ ο ∷ ύ ∷ τ ∷ ο ∷ υ ∷ []) "John.16.19"
∷ word (ζ ∷ η ∷ τ ∷ ε ∷ ῖ ∷ τ ∷ ε ∷ []) "John.16.19"
∷ word (μ ∷ ε ∷ τ ∷ []) "John.16.19"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ή ∷ ∙λ ∷ ω ∷ ν ∷ []) "John.16.19"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.16.19"
∷ word (ε ∷ ἶ ∷ π ∷ ο ∷ ν ∷ []) "John.16.19"
∷ word (Μ ∷ ι ∷ κ ∷ ρ ∷ ὸ ∷ ν ∷ []) "John.16.19"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.16.19"
∷ word (ο ∷ ὐ ∷ []) "John.16.19"
∷ word (θ ∷ ε ∷ ω ∷ ρ ∷ ε ∷ ῖ ∷ τ ∷ έ ∷ []) "John.16.19"
∷ word (μ ∷ ε ∷ []) "John.16.19"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.16.19"
∷ word (π ∷ ά ∷ ∙λ ∷ ι ∷ ν ∷ []) "John.16.19"
∷ word (μ ∷ ι ∷ κ ∷ ρ ∷ ὸ ∷ ν ∷ []) "John.16.19"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.16.19"
∷ word (ὄ ∷ ψ ∷ ε ∷ σ ∷ θ ∷ έ ∷ []) "John.16.19"
∷ word (μ ∷ ε ∷ []) "John.16.19"
∷ word (ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.16.20"
∷ word (ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.16.20"
∷ word (∙λ ∷ έ ∷ γ ∷ ω ∷ []) "John.16.20"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.16.20"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.16.20"
∷ word (κ ∷ ∙λ ∷ α ∷ ύ ∷ σ ∷ ε ∷ τ ∷ ε ∷ []) "John.16.20"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.16.20"
∷ word (θ ∷ ρ ∷ η ∷ ν ∷ ή ∷ σ ∷ ε ∷ τ ∷ ε ∷ []) "John.16.20"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.16.20"
∷ word (ὁ ∷ []) "John.16.20"
∷ word (δ ∷ ὲ ∷ []) "John.16.20"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ ς ∷ []) "John.16.20"
∷ word (χ ∷ α ∷ ρ ∷ ή ∷ σ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.16.20"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.16.20"
∷ word (∙λ ∷ υ ∷ π ∷ η ∷ θ ∷ ή ∷ σ ∷ ε ∷ σ ∷ θ ∷ ε ∷ []) "John.16.20"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ []) "John.16.20"
∷ word (ἡ ∷ []) "John.16.20"
∷ word (∙λ ∷ ύ ∷ π ∷ η ∷ []) "John.16.20"
∷ word (ὑ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.16.20"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.16.20"
∷ word (χ ∷ α ∷ ρ ∷ ὰ ∷ ν ∷ []) "John.16.20"
∷ word (γ ∷ ε ∷ ν ∷ ή ∷ σ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.16.20"
∷ word (ἡ ∷ []) "John.16.21"
∷ word (γ ∷ υ ∷ ν ∷ ὴ ∷ []) "John.16.21"
∷ word (ὅ ∷ τ ∷ α ∷ ν ∷ []) "John.16.21"
∷ word (τ ∷ ί ∷ κ ∷ τ ∷ ῃ ∷ []) "John.16.21"
∷ word (∙λ ∷ ύ ∷ π ∷ η ∷ ν ∷ []) "John.16.21"
∷ word (ἔ ∷ χ ∷ ε ∷ ι ∷ []) "John.16.21"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.16.21"
∷ word (ἦ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.16.21"
∷ word (ἡ ∷ []) "John.16.21"
∷ word (ὥ ∷ ρ ∷ α ∷ []) "John.16.21"
∷ word (α ∷ ὐ ∷ τ ∷ ῆ ∷ ς ∷ []) "John.16.21"
∷ word (ὅ ∷ τ ∷ α ∷ ν ∷ []) "John.16.21"
∷ word (δ ∷ ὲ ∷ []) "John.16.21"
∷ word (γ ∷ ε ∷ ν ∷ ν ∷ ή ∷ σ ∷ ῃ ∷ []) "John.16.21"
∷ word (τ ∷ ὸ ∷ []) "John.16.21"
∷ word (π ∷ α ∷ ι ∷ δ ∷ ί ∷ ο ∷ ν ∷ []) "John.16.21"
∷ word (ο ∷ ὐ ∷ κ ∷ έ ∷ τ ∷ ι ∷ []) "John.16.21"
∷ word (μ ∷ ν ∷ η ∷ μ ∷ ο ∷ ν ∷ ε ∷ ύ ∷ ε ∷ ι ∷ []) "John.16.21"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.16.21"
∷ word (θ ∷ ∙λ ∷ ί ∷ ψ ∷ ε ∷ ω ∷ ς ∷ []) "John.16.21"
∷ word (δ ∷ ι ∷ ὰ ∷ []) "John.16.21"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.16.21"
∷ word (χ ∷ α ∷ ρ ∷ ὰ ∷ ν ∷ []) "John.16.21"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.16.21"
∷ word (ἐ ∷ γ ∷ ε ∷ ν ∷ ν ∷ ή ∷ θ ∷ η ∷ []) "John.16.21"
∷ word (ἄ ∷ ν ∷ θ ∷ ρ ∷ ω ∷ π ∷ ο ∷ ς ∷ []) "John.16.21"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.16.21"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.16.21"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ ν ∷ []) "John.16.21"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.16.22"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.16.22"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.16.22"
∷ word (ν ∷ ῦ ∷ ν ∷ []) "John.16.22"
∷ word (μ ∷ ὲ ∷ ν ∷ []) "John.16.22"
∷ word (∙λ ∷ ύ ∷ π ∷ η ∷ ν ∷ []) "John.16.22"
∷ word (ἔ ∷ χ ∷ ε ∷ τ ∷ ε ∷ []) "John.16.22"
∷ word (π ∷ ά ∷ ∙λ ∷ ι ∷ ν ∷ []) "John.16.22"
∷ word (δ ∷ ὲ ∷ []) "John.16.22"
∷ word (ὄ ∷ ψ ∷ ο ∷ μ ∷ α ∷ ι ∷ []) "John.16.22"
∷ word (ὑ ∷ μ ∷ ᾶ ∷ ς ∷ []) "John.16.22"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.16.22"
∷ word (χ ∷ α ∷ ρ ∷ ή ∷ σ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.16.22"
∷ word (ὑ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.16.22"
∷ word (ἡ ∷ []) "John.16.22"
∷ word (κ ∷ α ∷ ρ ∷ δ ∷ ί ∷ α ∷ []) "John.16.22"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.16.22"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.16.22"
∷ word (χ ∷ α ∷ ρ ∷ ὰ ∷ ν ∷ []) "John.16.22"
∷ word (ὑ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.16.22"
∷ word (ο ∷ ὐ ∷ δ ∷ ε ∷ ὶ ∷ ς ∷ []) "John.16.22"
∷ word (α ∷ ἴ ∷ ρ ∷ ε ∷ ι ∷ []) "John.16.22"
∷ word (ἀ ∷ φ ∷ []) "John.16.22"
∷ word (ὑ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.16.22"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.16.23"
∷ word (ἐ ∷ ν ∷ []) "John.16.23"
∷ word (ἐ ∷ κ ∷ ε ∷ ί ∷ ν ∷ ῃ ∷ []) "John.16.23"
∷ word (τ ∷ ῇ ∷ []) "John.16.23"
∷ word (ἡ ∷ μ ∷ έ ∷ ρ ∷ ᾳ ∷ []) "John.16.23"
∷ word (ἐ ∷ μ ∷ ὲ ∷ []) "John.16.23"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.16.23"
∷ word (ἐ ∷ ρ ∷ ω ∷ τ ∷ ή ∷ σ ∷ ε ∷ τ ∷ ε ∷ []) "John.16.23"
∷ word (ο ∷ ὐ ∷ δ ∷ έ ∷ ν ∷ []) "John.16.23"
∷ word (ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.16.23"
∷ word (ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.16.23"
∷ word (∙λ ∷ έ ∷ γ ∷ ω ∷ []) "John.16.23"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.16.23"
∷ word (ἄ ∷ ν ∷ []) "John.16.23"
∷ word (τ ∷ ι ∷ []) "John.16.23"
∷ word (α ∷ ἰ ∷ τ ∷ ή ∷ σ ∷ η ∷ τ ∷ ε ∷ []) "John.16.23"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.16.23"
∷ word (π ∷ α ∷ τ ∷ έ ∷ ρ ∷ α ∷ []) "John.16.23"
∷ word (δ ∷ ώ ∷ σ ∷ ε ∷ ι ∷ []) "John.16.23"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.16.23"
∷ word (ἐ ∷ ν ∷ []) "John.16.23"
∷ word (τ ∷ ῷ ∷ []) "John.16.23"
∷ word (ὀ ∷ ν ∷ ό ∷ μ ∷ α ∷ τ ∷ ί ∷ []) "John.16.23"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.16.23"
∷ word (ἕ ∷ ω ∷ ς ∷ []) "John.16.24"
∷ word (ἄ ∷ ρ ∷ τ ∷ ι ∷ []) "John.16.24"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.16.24"
∷ word (ᾐ ∷ τ ∷ ή ∷ σ ∷ α ∷ τ ∷ ε ∷ []) "John.16.24"
∷ word (ο ∷ ὐ ∷ δ ∷ ὲ ∷ ν ∷ []) "John.16.24"
∷ word (ἐ ∷ ν ∷ []) "John.16.24"
∷ word (τ ∷ ῷ ∷ []) "John.16.24"
∷ word (ὀ ∷ ν ∷ ό ∷ μ ∷ α ∷ τ ∷ ί ∷ []) "John.16.24"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.16.24"
∷ word (α ∷ ἰ ∷ τ ∷ ε ∷ ῖ ∷ τ ∷ ε ∷ []) "John.16.24"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.16.24"
∷ word (∙λ ∷ ή ∷ μ ∷ ψ ∷ ε ∷ σ ∷ θ ∷ ε ∷ []) "John.16.24"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.16.24"
∷ word (ἡ ∷ []) "John.16.24"
∷ word (χ ∷ α ∷ ρ ∷ ὰ ∷ []) "John.16.24"
∷ word (ὑ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.16.24"
∷ word (ᾖ ∷ []) "John.16.24"
∷ word (π ∷ ε ∷ π ∷ ∙λ ∷ η ∷ ρ ∷ ω ∷ μ ∷ έ ∷ ν ∷ η ∷ []) "John.16.24"
∷ word (Τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.16.25"
∷ word (ἐ ∷ ν ∷ []) "John.16.25"
∷ word (π ∷ α ∷ ρ ∷ ο ∷ ι ∷ μ ∷ ί ∷ α ∷ ι ∷ ς ∷ []) "John.16.25"
∷ word (∙λ ∷ ε ∷ ∙λ ∷ ά ∷ ∙λ ∷ η ∷ κ ∷ α ∷ []) "John.16.25"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.16.25"
∷ word (ἔ ∷ ρ ∷ χ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.16.25"
∷ word (ὥ ∷ ρ ∷ α ∷ []) "John.16.25"
∷ word (ὅ ∷ τ ∷ ε ∷ []) "John.16.25"
∷ word (ο ∷ ὐ ∷ κ ∷ έ ∷ τ ∷ ι ∷ []) "John.16.25"
∷ word (ἐ ∷ ν ∷ []) "John.16.25"
∷ word (π ∷ α ∷ ρ ∷ ο ∷ ι ∷ μ ∷ ί ∷ α ∷ ι ∷ ς ∷ []) "John.16.25"
∷ word (∙λ ∷ α ∷ ∙λ ∷ ή ∷ σ ∷ ω ∷ []) "John.16.25"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.16.25"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.16.25"
∷ word (π ∷ α ∷ ρ ∷ ρ ∷ η ∷ σ ∷ ί ∷ ᾳ ∷ []) "John.16.25"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.16.25"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.16.25"
∷ word (π ∷ α ∷ τ ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.16.25"
∷ word (ἀ ∷ π ∷ α ∷ γ ∷ γ ∷ ε ∷ ∙λ ∷ ῶ ∷ []) "John.16.25"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.16.25"
∷ word (ἐ ∷ ν ∷ []) "John.16.26"
∷ word (ἐ ∷ κ ∷ ε ∷ ί ∷ ν ∷ ῃ ∷ []) "John.16.26"
∷ word (τ ∷ ῇ ∷ []) "John.16.26"
∷ word (ἡ ∷ μ ∷ έ ∷ ρ ∷ ᾳ ∷ []) "John.16.26"
∷ word (ἐ ∷ ν ∷ []) "John.16.26"
∷ word (τ ∷ ῷ ∷ []) "John.16.26"
∷ word (ὀ ∷ ν ∷ ό ∷ μ ∷ α ∷ τ ∷ ί ∷ []) "John.16.26"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.16.26"
∷ word (α ∷ ἰ ∷ τ ∷ ή ∷ σ ∷ ε ∷ σ ∷ θ ∷ ε ∷ []) "John.16.26"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.16.26"
∷ word (ο ∷ ὐ ∷ []) "John.16.26"
∷ word (∙λ ∷ έ ∷ γ ∷ ω ∷ []) "John.16.26"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.16.26"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.16.26"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.16.26"
∷ word (ἐ ∷ ρ ∷ ω ∷ τ ∷ ή ∷ σ ∷ ω ∷ []) "John.16.26"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.16.26"
∷ word (π ∷ α ∷ τ ∷ έ ∷ ρ ∷ α ∷ []) "John.16.26"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.16.26"
∷ word (ὑ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.16.26"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ς ∷ []) "John.16.27"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.16.27"
∷ word (ὁ ∷ []) "John.16.27"
∷ word (π ∷ α ∷ τ ∷ ὴ ∷ ρ ∷ []) "John.16.27"
∷ word (φ ∷ ι ∷ ∙λ ∷ ε ∷ ῖ ∷ []) "John.16.27"
∷ word (ὑ ∷ μ ∷ ᾶ ∷ ς ∷ []) "John.16.27"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.16.27"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.16.27"
∷ word (ἐ ∷ μ ∷ ὲ ∷ []) "John.16.27"
∷ word (π ∷ ε ∷ φ ∷ ι ∷ ∙λ ∷ ή ∷ κ ∷ α ∷ τ ∷ ε ∷ []) "John.16.27"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.16.27"
∷ word (π ∷ ε ∷ π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ κ ∷ α ∷ τ ∷ ε ∷ []) "John.16.27"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.16.27"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.16.27"
∷ word (π ∷ α ∷ ρ ∷ ὰ ∷ []) "John.16.27"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.16.27"
∷ word (θ ∷ ε ∷ ο ∷ ῦ ∷ []) "John.16.27"
∷ word (ἐ ∷ ξ ∷ ῆ ∷ ∙λ ∷ θ ∷ ο ∷ ν ∷ []) "John.16.27"
∷ word (ἐ ∷ ξ ∷ ῆ ∷ ∙λ ∷ θ ∷ ο ∷ ν ∷ []) "John.16.28"
∷ word (ἐ ∷ κ ∷ []) "John.16.28"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.16.28"
∷ word (π ∷ α ∷ τ ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.16.28"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.16.28"
∷ word (ἐ ∷ ∙λ ∷ ή ∷ ∙λ ∷ υ ∷ θ ∷ α ∷ []) "John.16.28"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.16.28"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.16.28"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ ν ∷ []) "John.16.28"
∷ word (π ∷ ά ∷ ∙λ ∷ ι ∷ ν ∷ []) "John.16.28"
∷ word (ἀ ∷ φ ∷ ί ∷ η ∷ μ ∷ ι ∷ []) "John.16.28"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.16.28"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ ν ∷ []) "John.16.28"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.16.28"
∷ word (π ∷ ο ∷ ρ ∷ ε ∷ ύ ∷ ο ∷ μ ∷ α ∷ ι ∷ []) "John.16.28"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.16.28"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.16.28"
∷ word (π ∷ α ∷ τ ∷ έ ∷ ρ ∷ α ∷ []) "John.16.28"
∷ word (Λ ∷ έ ∷ γ ∷ ο ∷ υ ∷ σ ∷ ι ∷ ν ∷ []) "John.16.29"
∷ word (ο ∷ ἱ ∷ []) "John.16.29"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ α ∷ ὶ ∷ []) "John.16.29"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.16.29"
∷ word (Ἴ ∷ δ ∷ ε ∷ []) "John.16.29"
∷ word (ν ∷ ῦ ∷ ν ∷ []) "John.16.29"
∷ word (ἐ ∷ ν ∷ []) "John.16.29"
∷ word (π ∷ α ∷ ρ ∷ ρ ∷ η ∷ σ ∷ ί ∷ ᾳ ∷ []) "John.16.29"
∷ word (∙λ ∷ α ∷ ∙λ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.16.29"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.16.29"
∷ word (π ∷ α ∷ ρ ∷ ο ∷ ι ∷ μ ∷ ί ∷ α ∷ ν ∷ []) "John.16.29"
∷ word (ο ∷ ὐ ∷ δ ∷ ε ∷ μ ∷ ί ∷ α ∷ ν ∷ []) "John.16.29"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ ς ∷ []) "John.16.29"
∷ word (ν ∷ ῦ ∷ ν ∷ []) "John.16.30"
∷ word (ο ∷ ἴ ∷ δ ∷ α ∷ μ ∷ ε ∷ ν ∷ []) "John.16.30"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.16.30"
∷ word (ο ∷ ἶ ∷ δ ∷ α ∷ ς ∷ []) "John.16.30"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ α ∷ []) "John.16.30"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.16.30"
∷ word (ο ∷ ὐ ∷ []) "John.16.30"
∷ word (χ ∷ ρ ∷ ε ∷ ί ∷ α ∷ ν ∷ []) "John.16.30"
∷ word (ἔ ∷ χ ∷ ε ∷ ι ∷ ς ∷ []) "John.16.30"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.16.30"
∷ word (τ ∷ ί ∷ ς ∷ []) "John.16.30"
∷ word (σ ∷ ε ∷ []) "John.16.30"
∷ word (ἐ ∷ ρ ∷ ω ∷ τ ∷ ᾷ ∷ []) "John.16.30"
∷ word (ἐ ∷ ν ∷ []) "John.16.30"
∷ word (τ ∷ ο ∷ ύ ∷ τ ∷ ῳ ∷ []) "John.16.30"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ ο ∷ μ ∷ ε ∷ ν ∷ []) "John.16.30"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.16.30"
∷ word (ἀ ∷ π ∷ ὸ ∷ []) "John.16.30"
∷ word (θ ∷ ε ∷ ο ∷ ῦ ∷ []) "John.16.30"
∷ word (ἐ ∷ ξ ∷ ῆ ∷ ∙λ ∷ θ ∷ ε ∷ ς ∷ []) "John.16.30"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.16.31"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.16.31"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.16.31"
∷ word (Ἄ ∷ ρ ∷ τ ∷ ι ∷ []) "John.16.31"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ ε ∷ τ ∷ ε ∷ []) "John.16.31"
∷ word (ἰ ∷ δ ∷ ο ∷ ὺ ∷ []) "John.16.32"
∷ word (ἔ ∷ ρ ∷ χ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.16.32"
∷ word (ὥ ∷ ρ ∷ α ∷ []) "John.16.32"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.16.32"
∷ word (ἐ ∷ ∙λ ∷ ή ∷ ∙λ ∷ υ ∷ θ ∷ ε ∷ ν ∷ []) "John.16.32"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.16.32"
∷ word (σ ∷ κ ∷ ο ∷ ρ ∷ π ∷ ι ∷ σ ∷ θ ∷ ῆ ∷ τ ∷ ε ∷ []) "John.16.32"
∷ word (ἕ ∷ κ ∷ α ∷ σ ∷ τ ∷ ο ∷ ς ∷ []) "John.16.32"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.16.32"
∷ word (τ ∷ ὰ ∷ []) "John.16.32"
∷ word (ἴ ∷ δ ∷ ι ∷ α ∷ []) "John.16.32"
∷ word (κ ∷ ἀ ∷ μ ∷ ὲ ∷ []) "John.16.32"
∷ word (μ ∷ ό ∷ ν ∷ ο ∷ ν ∷ []) "John.16.32"
∷ word (ἀ ∷ φ ∷ ῆ ∷ τ ∷ ε ∷ []) "John.16.32"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.16.32"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.16.32"
∷ word (ε ∷ ἰ ∷ μ ∷ ὶ ∷ []) "John.16.32"
∷ word (μ ∷ ό ∷ ν ∷ ο ∷ ς ∷ []) "John.16.32"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.16.32"
∷ word (ὁ ∷ []) "John.16.32"
∷ word (π ∷ α ∷ τ ∷ ὴ ∷ ρ ∷ []) "John.16.32"
∷ word (μ ∷ ε ∷ τ ∷ []) "John.16.32"
∷ word (ἐ ∷ μ ∷ ο ∷ ῦ ∷ []) "John.16.32"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.16.32"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.16.33"
∷ word (∙λ ∷ ε ∷ ∙λ ∷ ά ∷ ∙λ ∷ η ∷ κ ∷ α ∷ []) "John.16.33"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.16.33"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.16.33"
∷ word (ἐ ∷ ν ∷ []) "John.16.33"
∷ word (ἐ ∷ μ ∷ ο ∷ ὶ ∷ []) "John.16.33"
∷ word (ε ∷ ἰ ∷ ρ ∷ ή ∷ ν ∷ η ∷ ν ∷ []) "John.16.33"
∷ word (ἔ ∷ χ ∷ η ∷ τ ∷ ε ∷ []) "John.16.33"
∷ word (ἐ ∷ ν ∷ []) "John.16.33"
∷ word (τ ∷ ῷ ∷ []) "John.16.33"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ῳ ∷ []) "John.16.33"
∷ word (θ ∷ ∙λ ∷ ῖ ∷ ψ ∷ ι ∷ ν ∷ []) "John.16.33"
∷ word (ἔ ∷ χ ∷ ε ∷ τ ∷ ε ∷ []) "John.16.33"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.16.33"
∷ word (θ ∷ α ∷ ρ ∷ σ ∷ ε ∷ ῖ ∷ τ ∷ ε ∷ []) "John.16.33"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.16.33"
∷ word (ν ∷ ε ∷ ν ∷ ί ∷ κ ∷ η ∷ κ ∷ α ∷ []) "John.16.33"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.16.33"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ ν ∷ []) "John.16.33"
∷ word (Τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.17.1"
∷ word (ἐ ∷ ∙λ ∷ ά ∷ ∙λ ∷ η ∷ σ ∷ ε ∷ ν ∷ []) "John.17.1"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.17.1"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.17.1"
∷ word (ἐ ∷ π ∷ ά ∷ ρ ∷ α ∷ ς ∷ []) "John.17.1"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.17.1"
∷ word (ὀ ∷ φ ∷ θ ∷ α ∷ ∙λ ∷ μ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.17.1"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.17.1"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.17.1"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.17.1"
∷ word (ο ∷ ὐ ∷ ρ ∷ α ∷ ν ∷ ὸ ∷ ν ∷ []) "John.17.1"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.17.1"
∷ word (Π ∷ ά ∷ τ ∷ ε ∷ ρ ∷ []) "John.17.1"
∷ word (ἐ ∷ ∙λ ∷ ή ∷ ∙λ ∷ υ ∷ θ ∷ ε ∷ ν ∷ []) "John.17.1"
∷ word (ἡ ∷ []) "John.17.1"
∷ word (ὥ ∷ ρ ∷ α ∷ []) "John.17.1"
∷ word (δ ∷ ό ∷ ξ ∷ α ∷ σ ∷ ό ∷ ν ∷ []) "John.17.1"
∷ word (σ ∷ ο ∷ υ ∷ []) "John.17.1"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.17.1"
∷ word (υ ∷ ἱ ∷ ό ∷ ν ∷ []) "John.17.1"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.17.1"
∷ word (ὁ ∷ []) "John.17.1"
∷ word (υ ∷ ἱ ∷ ὸ ∷ ς ∷ []) "John.17.1"
∷ word (δ ∷ ο ∷ ξ ∷ ά ∷ σ ∷ ῃ ∷ []) "John.17.1"
∷ word (σ ∷ έ ∷ []) "John.17.1"
∷ word (κ ∷ α ∷ θ ∷ ὼ ∷ ς ∷ []) "John.17.2"
∷ word (ἔ ∷ δ ∷ ω ∷ κ ∷ α ∷ ς ∷ []) "John.17.2"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.17.2"
∷ word (ἐ ∷ ξ ∷ ο ∷ υ ∷ σ ∷ ί ∷ α ∷ ν ∷ []) "John.17.2"
∷ word (π ∷ ά ∷ σ ∷ η ∷ ς ∷ []) "John.17.2"
∷ word (σ ∷ α ∷ ρ ∷ κ ∷ ό ∷ ς ∷ []) "John.17.2"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.17.2"
∷ word (π ∷ ᾶ ∷ ν ∷ []) "John.17.2"
∷ word (ὃ ∷ []) "John.17.2"
∷ word (δ ∷ έ ∷ δ ∷ ω ∷ κ ∷ α ∷ ς ∷ []) "John.17.2"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.17.2"
∷ word (δ ∷ ώ ∷ σ ∷ ῃ ∷ []) "John.17.2"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.17.2"
∷ word (ζ ∷ ω ∷ ὴ ∷ ν ∷ []) "John.17.2"
∷ word (α ∷ ἰ ∷ ώ ∷ ν ∷ ι ∷ ο ∷ ν ∷ []) "John.17.2"
∷ word (α ∷ ὕ ∷ τ ∷ η ∷ []) "John.17.3"
∷ word (δ ∷ έ ∷ []) "John.17.3"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.17.3"
∷ word (ἡ ∷ []) "John.17.3"
∷ word (α ∷ ἰ ∷ ώ ∷ ν ∷ ι ∷ ο ∷ ς ∷ []) "John.17.3"
∷ word (ζ ∷ ω ∷ ὴ ∷ []) "John.17.3"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.17.3"
∷ word (γ ∷ ι ∷ ν ∷ ώ ∷ σ ∷ κ ∷ ω ∷ σ ∷ ι ∷ []) "John.17.3"
∷ word (σ ∷ ὲ ∷ []) "John.17.3"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.17.3"
∷ word (μ ∷ ό ∷ ν ∷ ο ∷ ν ∷ []) "John.17.3"
∷ word (ἀ ∷ ∙λ ∷ η ∷ θ ∷ ι ∷ ν ∷ ὸ ∷ ν ∷ []) "John.17.3"
∷ word (θ ∷ ε ∷ ὸ ∷ ν ∷ []) "John.17.3"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.17.3"
∷ word (ὃ ∷ ν ∷ []) "John.17.3"
∷ word (ἀ ∷ π ∷ έ ∷ σ ∷ τ ∷ ε ∷ ι ∷ ∙λ ∷ α ∷ ς ∷ []) "John.17.3"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ν ∷ []) "John.17.3"
∷ word (Χ ∷ ρ ∷ ι ∷ σ ∷ τ ∷ ό ∷ ν ∷ []) "John.17.3"
∷ word (ἐ ∷ γ ∷ ώ ∷ []) "John.17.4"
∷ word (σ ∷ ε ∷ []) "John.17.4"
∷ word (ἐ ∷ δ ∷ ό ∷ ξ ∷ α ∷ σ ∷ α ∷ []) "John.17.4"
∷ word (ἐ ∷ π ∷ ὶ ∷ []) "John.17.4"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.17.4"
∷ word (γ ∷ ῆ ∷ ς ∷ []) "John.17.4"
∷ word (τ ∷ ὸ ∷ []) "John.17.4"
∷ word (ἔ ∷ ρ ∷ γ ∷ ο ∷ ν ∷ []) "John.17.4"
∷ word (τ ∷ ε ∷ ∙λ ∷ ε ∷ ι ∷ ώ ∷ σ ∷ α ∷ ς ∷ []) "John.17.4"
∷ word (ὃ ∷ []) "John.17.4"
∷ word (δ ∷ έ ∷ δ ∷ ω ∷ κ ∷ ά ∷ ς ∷ []) "John.17.4"
∷ word (μ ∷ ο ∷ ι ∷ []) "John.17.4"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.17.4"
∷ word (π ∷ ο ∷ ι ∷ ή ∷ σ ∷ ω ∷ []) "John.17.4"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.17.5"
∷ word (ν ∷ ῦ ∷ ν ∷ []) "John.17.5"
∷ word (δ ∷ ό ∷ ξ ∷ α ∷ σ ∷ ό ∷ ν ∷ []) "John.17.5"
∷ word (μ ∷ ε ∷ []) "John.17.5"
∷ word (σ ∷ ύ ∷ []) "John.17.5"
∷ word (π ∷ ά ∷ τ ∷ ε ∷ ρ ∷ []) "John.17.5"
∷ word (π ∷ α ∷ ρ ∷ ὰ ∷ []) "John.17.5"
∷ word (σ ∷ ε ∷ α ∷ υ ∷ τ ∷ ῷ ∷ []) "John.17.5"
∷ word (τ ∷ ῇ ∷ []) "John.17.5"
∷ word (δ ∷ ό ∷ ξ ∷ ῃ ∷ []) "John.17.5"
∷ word (ᾗ ∷ []) "John.17.5"
∷ word (ε ∷ ἶ ∷ χ ∷ ο ∷ ν ∷ []) "John.17.5"
∷ word (π ∷ ρ ∷ ὸ ∷ []) "John.17.5"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.17.5"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.17.5"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ ν ∷ []) "John.17.5"
∷ word (ε ∷ ἶ ∷ ν ∷ α ∷ ι ∷ []) "John.17.5"
∷ word (π ∷ α ∷ ρ ∷ ὰ ∷ []) "John.17.5"
∷ word (σ ∷ ο ∷ ί ∷ []) "John.17.5"
∷ word (Ἐ ∷ φ ∷ α ∷ ν ∷ έ ∷ ρ ∷ ω ∷ σ ∷ ά ∷ []) "John.17.6"
∷ word (σ ∷ ο ∷ υ ∷ []) "John.17.6"
∷ word (τ ∷ ὸ ∷ []) "John.17.6"
∷ word (ὄ ∷ ν ∷ ο ∷ μ ∷ α ∷ []) "John.17.6"
∷ word (τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.17.6"
∷ word (ἀ ∷ ν ∷ θ ∷ ρ ∷ ώ ∷ π ∷ ο ∷ ι ∷ ς ∷ []) "John.17.6"
∷ word (ο ∷ ὓ ∷ ς ∷ []) "John.17.6"
∷ word (ἔ ∷ δ ∷ ω ∷ κ ∷ ά ∷ ς ∷ []) "John.17.6"
∷ word (μ ∷ ο ∷ ι ∷ []) "John.17.6"
∷ word (ἐ ∷ κ ∷ []) "John.17.6"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.17.6"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ υ ∷ []) "John.17.6"
∷ word (σ ∷ ο ∷ ὶ ∷ []) "John.17.6"
∷ word (ἦ ∷ σ ∷ α ∷ ν ∷ []) "John.17.6"
∷ word (κ ∷ ἀ ∷ μ ∷ ο ∷ ὶ ∷ []) "John.17.6"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.17.6"
∷ word (ἔ ∷ δ ∷ ω ∷ κ ∷ α ∷ ς ∷ []) "John.17.6"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.17.6"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.17.6"
∷ word (∙λ ∷ ό ∷ γ ∷ ο ∷ ν ∷ []) "John.17.6"
∷ word (σ ∷ ο ∷ υ ∷ []) "John.17.6"
∷ word (τ ∷ ε ∷ τ ∷ ή ∷ ρ ∷ η ∷ κ ∷ α ∷ ν ∷ []) "John.17.6"
∷ word (ν ∷ ῦ ∷ ν ∷ []) "John.17.7"
∷ word (ἔ ∷ γ ∷ ν ∷ ω ∷ κ ∷ α ∷ ν ∷ []) "John.17.7"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.17.7"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ α ∷ []) "John.17.7"
∷ word (ὅ ∷ σ ∷ α ∷ []) "John.17.7"
∷ word (δ ∷ έ ∷ δ ∷ ω ∷ κ ∷ ά ∷ ς ∷ []) "John.17.7"
∷ word (μ ∷ ο ∷ ι ∷ []) "John.17.7"
∷ word (π ∷ α ∷ ρ ∷ ὰ ∷ []) "John.17.7"
∷ word (σ ∷ ο ∷ ῦ ∷ []) "John.17.7"
∷ word (ε ∷ ἰ ∷ σ ∷ ι ∷ ν ∷ []) "John.17.7"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.17.8"
∷ word (τ ∷ ὰ ∷ []) "John.17.8"
∷ word (ῥ ∷ ή ∷ μ ∷ α ∷ τ ∷ α ∷ []) "John.17.8"
∷ word (ἃ ∷ []) "John.17.8"
∷ word (ἔ ∷ δ ∷ ω ∷ κ ∷ ά ∷ ς ∷ []) "John.17.8"
∷ word (μ ∷ ο ∷ ι ∷ []) "John.17.8"
∷ word (δ ∷ έ ∷ δ ∷ ω ∷ κ ∷ α ∷ []) "John.17.8"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.17.8"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.17.8"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ὶ ∷ []) "John.17.8"
∷ word (ἔ ∷ ∙λ ∷ α ∷ β ∷ ο ∷ ν ∷ []) "John.17.8"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.17.8"
∷ word (ἔ ∷ γ ∷ ν ∷ ω ∷ σ ∷ α ∷ ν ∷ []) "John.17.8"
∷ word (ἀ ∷ ∙λ ∷ η ∷ θ ∷ ῶ ∷ ς ∷ []) "John.17.8"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.17.8"
∷ word (π ∷ α ∷ ρ ∷ ὰ ∷ []) "John.17.8"
∷ word (σ ∷ ο ∷ ῦ ∷ []) "John.17.8"
∷ word (ἐ ∷ ξ ∷ ῆ ∷ ∙λ ∷ θ ∷ ο ∷ ν ∷ []) "John.17.8"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.17.8"
∷ word (ἐ ∷ π ∷ ί ∷ σ ∷ τ ∷ ε ∷ υ ∷ σ ∷ α ∷ ν ∷ []) "John.17.8"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.17.8"
∷ word (σ ∷ ύ ∷ []) "John.17.8"
∷ word (μ ∷ ε ∷ []) "John.17.8"
∷ word (ἀ ∷ π ∷ έ ∷ σ ∷ τ ∷ ε ∷ ι ∷ ∙λ ∷ α ∷ ς ∷ []) "John.17.8"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.17.9"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.17.9"
∷ word (α ∷ ὐ ∷ τ ∷ ῶ ∷ ν ∷ []) "John.17.9"
∷ word (ἐ ∷ ρ ∷ ω ∷ τ ∷ ῶ ∷ []) "John.17.9"
∷ word (ο ∷ ὐ ∷ []) "John.17.9"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.17.9"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.17.9"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ υ ∷ []) "John.17.9"
∷ word (ἐ ∷ ρ ∷ ω ∷ τ ∷ ῶ ∷ []) "John.17.9"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.17.9"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.17.9"
∷ word (ὧ ∷ ν ∷ []) "John.17.9"
∷ word (δ ∷ έ ∷ δ ∷ ω ∷ κ ∷ ά ∷ ς ∷ []) "John.17.9"
∷ word (μ ∷ ο ∷ ι ∷ []) "John.17.9"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.17.9"
∷ word (σ ∷ ο ∷ ί ∷ []) "John.17.9"
∷ word (ε ∷ ἰ ∷ σ ∷ ι ∷ ν ∷ []) "John.17.9"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.17.10"
∷ word (τ ∷ ὰ ∷ []) "John.17.10"
∷ word (ἐ ∷ μ ∷ ὰ ∷ []) "John.17.10"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ α ∷ []) "John.17.10"
∷ word (σ ∷ ά ∷ []) "John.17.10"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.17.10"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.17.10"
∷ word (τ ∷ ὰ ∷ []) "John.17.10"
∷ word (σ ∷ ὰ ∷ []) "John.17.10"
∷ word (ἐ ∷ μ ∷ ά ∷ []) "John.17.10"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.17.10"
∷ word (δ ∷ ε ∷ δ ∷ ό ∷ ξ ∷ α ∷ σ ∷ μ ∷ α ∷ ι ∷ []) "John.17.10"
∷ word (ἐ ∷ ν ∷ []) "John.17.10"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.17.10"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.17.11"
∷ word (ο ∷ ὐ ∷ κ ∷ έ ∷ τ ∷ ι ∷ []) "John.17.11"
∷ word (ε ∷ ἰ ∷ μ ∷ ὶ ∷ []) "John.17.11"
∷ word (ἐ ∷ ν ∷ []) "John.17.11"
∷ word (τ ∷ ῷ ∷ []) "John.17.11"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ῳ ∷ []) "John.17.11"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.17.11"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ὶ ∷ []) "John.17.11"
∷ word (ἐ ∷ ν ∷ []) "John.17.11"
∷ word (τ ∷ ῷ ∷ []) "John.17.11"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ῳ ∷ []) "John.17.11"
∷ word (ε ∷ ἰ ∷ σ ∷ ί ∷ ν ∷ []) "John.17.11"
∷ word (κ ∷ ἀ ∷ γ ∷ ὼ ∷ []) "John.17.11"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.17.11"
∷ word (σ ∷ ὲ ∷ []) "John.17.11"
∷ word (ἔ ∷ ρ ∷ χ ∷ ο ∷ μ ∷ α ∷ ι ∷ []) "John.17.11"
∷ word (π ∷ ά ∷ τ ∷ ε ∷ ρ ∷ []) "John.17.11"
∷ word (ἅ ∷ γ ∷ ι ∷ ε ∷ []) "John.17.11"
∷ word (τ ∷ ή ∷ ρ ∷ η ∷ σ ∷ ο ∷ ν ∷ []) "John.17.11"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.17.11"
∷ word (ἐ ∷ ν ∷ []) "John.17.11"
∷ word (τ ∷ ῷ ∷ []) "John.17.11"
∷ word (ὀ ∷ ν ∷ ό ∷ μ ∷ α ∷ τ ∷ ί ∷ []) "John.17.11"
∷ word (σ ∷ ο ∷ υ ∷ []) "John.17.11"
∷ word (ᾧ ∷ []) "John.17.11"
∷ word (δ ∷ έ ∷ δ ∷ ω ∷ κ ∷ ά ∷ ς ∷ []) "John.17.11"
∷ word (μ ∷ ο ∷ ι ∷ []) "John.17.11"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.17.11"
∷ word (ὦ ∷ σ ∷ ι ∷ ν ∷ []) "John.17.11"
∷ word (ἓ ∷ ν ∷ []) "John.17.11"
∷ word (κ ∷ α ∷ θ ∷ ὼ ∷ ς ∷ []) "John.17.11"
∷ word (ἡ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.17.11"
∷ word (ὅ ∷ τ ∷ ε ∷ []) "John.17.12"
∷ word (ἤ ∷ μ ∷ η ∷ ν ∷ []) "John.17.12"
∷ word (μ ∷ ε ∷ τ ∷ []) "John.17.12"
∷ word (α ∷ ὐ ∷ τ ∷ ῶ ∷ ν ∷ []) "John.17.12"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.17.12"
∷ word (ἐ ∷ τ ∷ ή ∷ ρ ∷ ο ∷ υ ∷ ν ∷ []) "John.17.12"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.17.12"
∷ word (ἐ ∷ ν ∷ []) "John.17.12"
∷ word (τ ∷ ῷ ∷ []) "John.17.12"
∷ word (ὀ ∷ ν ∷ ό ∷ μ ∷ α ∷ τ ∷ ί ∷ []) "John.17.12"
∷ word (σ ∷ ο ∷ υ ∷ []) "John.17.12"
∷ word (ᾧ ∷ []) "John.17.12"
∷ word (δ ∷ έ ∷ δ ∷ ω ∷ κ ∷ ά ∷ ς ∷ []) "John.17.12"
∷ word (μ ∷ ο ∷ ι ∷ []) "John.17.12"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.17.12"
∷ word (ἐ ∷ φ ∷ ύ ∷ ∙λ ∷ α ∷ ξ ∷ α ∷ []) "John.17.12"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.17.12"
∷ word (ο ∷ ὐ ∷ δ ∷ ε ∷ ὶ ∷ ς ∷ []) "John.17.12"
∷ word (ἐ ∷ ξ ∷ []) "John.17.12"
∷ word (α ∷ ὐ ∷ τ ∷ ῶ ∷ ν ∷ []) "John.17.12"
∷ word (ἀ ∷ π ∷ ώ ∷ ∙λ ∷ ε ∷ τ ∷ ο ∷ []) "John.17.12"
∷ word (ε ∷ ἰ ∷ []) "John.17.12"
∷ word (μ ∷ ὴ ∷ []) "John.17.12"
∷ word (ὁ ∷ []) "John.17.12"
∷ word (υ ∷ ἱ ∷ ὸ ∷ ς ∷ []) "John.17.12"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.17.12"
∷ word (ἀ ∷ π ∷ ω ∷ ∙λ ∷ ε ∷ ί ∷ α ∷ ς ∷ []) "John.17.12"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.17.12"
∷ word (ἡ ∷ []) "John.17.12"
∷ word (γ ∷ ρ ∷ α ∷ φ ∷ ὴ ∷ []) "John.17.12"
∷ word (π ∷ ∙λ ∷ η ∷ ρ ∷ ω ∷ θ ∷ ῇ ∷ []) "John.17.12"
∷ word (ν ∷ ῦ ∷ ν ∷ []) "John.17.13"
∷ word (δ ∷ ὲ ∷ []) "John.17.13"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.17.13"
∷ word (σ ∷ ὲ ∷ []) "John.17.13"
∷ word (ἔ ∷ ρ ∷ χ ∷ ο ∷ μ ∷ α ∷ ι ∷ []) "John.17.13"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.17.13"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.17.13"
∷ word (∙λ ∷ α ∷ ∙λ ∷ ῶ ∷ []) "John.17.13"
∷ word (ἐ ∷ ν ∷ []) "John.17.13"
∷ word (τ ∷ ῷ ∷ []) "John.17.13"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ῳ ∷ []) "John.17.13"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.17.13"
∷ word (ἔ ∷ χ ∷ ω ∷ σ ∷ ι ∷ ν ∷ []) "John.17.13"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.17.13"
∷ word (χ ∷ α ∷ ρ ∷ ὰ ∷ ν ∷ []) "John.17.13"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.17.13"
∷ word (ἐ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.17.13"
∷ word (π ∷ ε ∷ π ∷ ∙λ ∷ η ∷ ρ ∷ ω ∷ μ ∷ έ ∷ ν ∷ η ∷ ν ∷ []) "John.17.13"
∷ word (ἐ ∷ ν ∷ []) "John.17.13"
∷ word (ἑ ∷ α ∷ υ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.17.13"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.17.14"
∷ word (δ ∷ έ ∷ δ ∷ ω ∷ κ ∷ α ∷ []) "John.17.14"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.17.14"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.17.14"
∷ word (∙λ ∷ ό ∷ γ ∷ ο ∷ ν ∷ []) "John.17.14"
∷ word (σ ∷ ο ∷ υ ∷ []) "John.17.14"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.17.14"
∷ word (ὁ ∷ []) "John.17.14"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ ς ∷ []) "John.17.14"
∷ word (ἐ ∷ μ ∷ ί ∷ σ ∷ η ∷ σ ∷ ε ∷ ν ∷ []) "John.17.14"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ύ ∷ ς ∷ []) "John.17.14"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.17.14"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.17.14"
∷ word (ε ∷ ἰ ∷ σ ∷ ὶ ∷ ν ∷ []) "John.17.14"
∷ word (ἐ ∷ κ ∷ []) "John.17.14"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.17.14"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ υ ∷ []) "John.17.14"
∷ word (κ ∷ α ∷ θ ∷ ὼ ∷ ς ∷ []) "John.17.14"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.17.14"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.17.14"
∷ word (ε ∷ ἰ ∷ μ ∷ ὶ ∷ []) "John.17.14"
∷ word (ἐ ∷ κ ∷ []) "John.17.14"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.17.14"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ υ ∷ []) "John.17.14"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.17.15"
∷ word (ἐ ∷ ρ ∷ ω ∷ τ ∷ ῶ ∷ []) "John.17.15"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.17.15"
∷ word (ἄ ∷ ρ ∷ ῃ ∷ ς ∷ []) "John.17.15"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.17.15"
∷ word (ἐ ∷ κ ∷ []) "John.17.15"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.17.15"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ υ ∷ []) "John.17.15"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ []) "John.17.15"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.17.15"
∷ word (τ ∷ η ∷ ρ ∷ ή ∷ σ ∷ ῃ ∷ ς ∷ []) "John.17.15"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.17.15"
∷ word (ἐ ∷ κ ∷ []) "John.17.15"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.17.15"
∷ word (π ∷ ο ∷ ν ∷ η ∷ ρ ∷ ο ∷ ῦ ∷ []) "John.17.15"
∷ word (ἐ ∷ κ ∷ []) "John.17.16"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.17.16"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ υ ∷ []) "John.17.16"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.17.16"
∷ word (ε ∷ ἰ ∷ σ ∷ ὶ ∷ ν ∷ []) "John.17.16"
∷ word (κ ∷ α ∷ θ ∷ ὼ ∷ ς ∷ []) "John.17.16"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.17.16"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.17.16"
∷ word (ε ∷ ἰ ∷ μ ∷ ὶ ∷ []) "John.17.16"
∷ word (ἐ ∷ κ ∷ []) "John.17.16"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.17.16"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ υ ∷ []) "John.17.16"
∷ word (ἁ ∷ γ ∷ ί ∷ α ∷ σ ∷ ο ∷ ν ∷ []) "John.17.17"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.17.17"
∷ word (ἐ ∷ ν ∷ []) "John.17.17"
∷ word (τ ∷ ῇ ∷ []) "John.17.17"
∷ word (ἀ ∷ ∙λ ∷ η ∷ θ ∷ ε ∷ ί ∷ ᾳ ∷ []) "John.17.17"
∷ word (ὁ ∷ []) "John.17.17"
∷ word (∙λ ∷ ό ∷ γ ∷ ο ∷ ς ∷ []) "John.17.17"
∷ word (ὁ ∷ []) "John.17.17"
∷ word (σ ∷ ὸ ∷ ς ∷ []) "John.17.17"
∷ word (ἀ ∷ ∙λ ∷ ή ∷ θ ∷ ε ∷ ι ∷ ά ∷ []) "John.17.17"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.17.17"
∷ word (κ ∷ α ∷ θ ∷ ὼ ∷ ς ∷ []) "John.17.18"
∷ word (ἐ ∷ μ ∷ ὲ ∷ []) "John.17.18"
∷ word (ἀ ∷ π ∷ έ ∷ σ ∷ τ ∷ ε ∷ ι ∷ ∙λ ∷ α ∷ ς ∷ []) "John.17.18"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.17.18"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.17.18"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ ν ∷ []) "John.17.18"
∷ word (κ ∷ ἀ ∷ γ ∷ ὼ ∷ []) "John.17.18"
∷ word (ἀ ∷ π ∷ έ ∷ σ ∷ τ ∷ ε ∷ ι ∷ ∙λ ∷ α ∷ []) "John.17.18"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.17.18"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.17.18"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.17.18"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ ν ∷ []) "John.17.18"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.17.19"
∷ word (ὑ ∷ π ∷ ὲ ∷ ρ ∷ []) "John.17.19"
∷ word (α ∷ ὐ ∷ τ ∷ ῶ ∷ ν ∷ []) "John.17.19"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.17.19"
∷ word (ἁ ∷ γ ∷ ι ∷ ά ∷ ζ ∷ ω ∷ []) "John.17.19"
∷ word (ἐ ∷ μ ∷ α ∷ υ ∷ τ ∷ ό ∷ ν ∷ []) "John.17.19"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.17.19"
∷ word (ὦ ∷ σ ∷ ι ∷ ν ∷ []) "John.17.19"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.17.19"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ὶ ∷ []) "John.17.19"
∷ word (ἡ ∷ γ ∷ ι ∷ α ∷ σ ∷ μ ∷ έ ∷ ν ∷ ο ∷ ι ∷ []) "John.17.19"
∷ word (ἐ ∷ ν ∷ []) "John.17.19"
∷ word (ἀ ∷ ∙λ ∷ η ∷ θ ∷ ε ∷ ί ∷ ᾳ ∷ []) "John.17.19"
∷ word (Ο ∷ ὐ ∷ []) "John.17.20"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.17.20"
∷ word (τ ∷ ο ∷ ύ ∷ τ ∷ ω ∷ ν ∷ []) "John.17.20"
∷ word (δ ∷ ὲ ∷ []) "John.17.20"
∷ word (ἐ ∷ ρ ∷ ω ∷ τ ∷ ῶ ∷ []) "John.17.20"
∷ word (μ ∷ ό ∷ ν ∷ ο ∷ ν ∷ []) "John.17.20"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.17.20"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.17.20"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.17.20"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.17.20"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ υ ∷ ό ∷ ν ∷ τ ∷ ω ∷ ν ∷ []) "John.17.20"
∷ word (δ ∷ ι ∷ ὰ ∷ []) "John.17.20"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.17.20"
∷ word (∙λ ∷ ό ∷ γ ∷ ο ∷ υ ∷ []) "John.17.20"
∷ word (α ∷ ὐ ∷ τ ∷ ῶ ∷ ν ∷ []) "John.17.20"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.17.20"
∷ word (ἐ ∷ μ ∷ έ ∷ []) "John.17.20"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.17.21"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.17.21"
∷ word (ἓ ∷ ν ∷ []) "John.17.21"
∷ word (ὦ ∷ σ ∷ ι ∷ ν ∷ []) "John.17.21"
∷ word (κ ∷ α ∷ θ ∷ ὼ ∷ ς ∷ []) "John.17.21"
∷ word (σ ∷ ύ ∷ []) "John.17.21"
∷ word (π ∷ ά ∷ τ ∷ ε ∷ ρ ∷ []) "John.17.21"
∷ word (ἐ ∷ ν ∷ []) "John.17.21"
∷ word (ἐ ∷ μ ∷ ο ∷ ὶ ∷ []) "John.17.21"
∷ word (κ ∷ ἀ ∷ γ ∷ ὼ ∷ []) "John.17.21"
∷ word (ἐ ∷ ν ∷ []) "John.17.21"
∷ word (σ ∷ ο ∷ ί ∷ []) "John.17.21"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.17.21"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.17.21"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ὶ ∷ []) "John.17.21"
∷ word (ἐ ∷ ν ∷ []) "John.17.21"
∷ word (ἡ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.17.21"
∷ word (ὦ ∷ σ ∷ ι ∷ ν ∷ []) "John.17.21"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.17.21"
∷ word (ὁ ∷ []) "John.17.21"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ ς ∷ []) "John.17.21"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ ῃ ∷ []) "John.17.21"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.17.21"
∷ word (σ ∷ ύ ∷ []) "John.17.21"
∷ word (μ ∷ ε ∷ []) "John.17.21"
∷ word (ἀ ∷ π ∷ έ ∷ σ ∷ τ ∷ ε ∷ ι ∷ ∙λ ∷ α ∷ ς ∷ []) "John.17.21"
∷ word (κ ∷ ἀ ∷ γ ∷ ὼ ∷ []) "John.17.22"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.17.22"
∷ word (δ ∷ ό ∷ ξ ∷ α ∷ ν ∷ []) "John.17.22"
∷ word (ἣ ∷ ν ∷ []) "John.17.22"
∷ word (δ ∷ έ ∷ δ ∷ ω ∷ κ ∷ ά ∷ ς ∷ []) "John.17.22"
∷ word (μ ∷ ο ∷ ι ∷ []) "John.17.22"
∷ word (δ ∷ έ ∷ δ ∷ ω ∷ κ ∷ α ∷ []) "John.17.22"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.17.22"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.17.22"
∷ word (ὦ ∷ σ ∷ ι ∷ ν ∷ []) "John.17.22"
∷ word (ἓ ∷ ν ∷ []) "John.17.22"
∷ word (κ ∷ α ∷ θ ∷ ὼ ∷ ς ∷ []) "John.17.22"
∷ word (ἡ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.17.22"
∷ word (ἕ ∷ ν ∷ []) "John.17.22"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.17.23"
∷ word (ἐ ∷ ν ∷ []) "John.17.23"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.17.23"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.17.23"
∷ word (σ ∷ ὺ ∷ []) "John.17.23"
∷ word (ἐ ∷ ν ∷ []) "John.17.23"
∷ word (ἐ ∷ μ ∷ ο ∷ ί ∷ []) "John.17.23"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.17.23"
∷ word (ὦ ∷ σ ∷ ι ∷ ν ∷ []) "John.17.23"
∷ word (τ ∷ ε ∷ τ ∷ ε ∷ ∙λ ∷ ε ∷ ι ∷ ω ∷ μ ∷ έ ∷ ν ∷ ο ∷ ι ∷ []) "John.17.23"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.17.23"
∷ word (ἕ ∷ ν ∷ []) "John.17.23"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.17.23"
∷ word (γ ∷ ι ∷ ν ∷ ώ ∷ σ ∷ κ ∷ ῃ ∷ []) "John.17.23"
∷ word (ὁ ∷ []) "John.17.23"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ ς ∷ []) "John.17.23"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.17.23"
∷ word (σ ∷ ύ ∷ []) "John.17.23"
∷ word (μ ∷ ε ∷ []) "John.17.23"
∷ word (ἀ ∷ π ∷ έ ∷ σ ∷ τ ∷ ε ∷ ι ∷ ∙λ ∷ α ∷ ς ∷ []) "John.17.23"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.17.23"
∷ word (ἠ ∷ γ ∷ ά ∷ π ∷ η ∷ σ ∷ α ∷ ς ∷ []) "John.17.23"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.17.23"
∷ word (κ ∷ α ∷ θ ∷ ὼ ∷ ς ∷ []) "John.17.23"
∷ word (ἐ ∷ μ ∷ ὲ ∷ []) "John.17.23"
∷ word (ἠ ∷ γ ∷ ά ∷ π ∷ η ∷ σ ∷ α ∷ ς ∷ []) "John.17.23"
∷ word (π ∷ ά ∷ τ ∷ ε ∷ ρ ∷ []) "John.17.24"
∷ word (ὃ ∷ []) "John.17.24"
∷ word (δ ∷ έ ∷ δ ∷ ω ∷ κ ∷ ά ∷ ς ∷ []) "John.17.24"
∷ word (μ ∷ ο ∷ ι ∷ []) "John.17.24"
∷ word (θ ∷ έ ∷ ∙λ ∷ ω ∷ []) "John.17.24"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.17.24"
∷ word (ὅ ∷ π ∷ ο ∷ υ ∷ []) "John.17.24"
∷ word (ε ∷ ἰ ∷ μ ∷ ὶ ∷ []) "John.17.24"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.17.24"
∷ word (κ ∷ ἀ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ο ∷ ι ∷ []) "John.17.24"
∷ word (ὦ ∷ σ ∷ ι ∷ ν ∷ []) "John.17.24"
∷ word (μ ∷ ε ∷ τ ∷ []) "John.17.24"
∷ word (ἐ ∷ μ ∷ ο ∷ ῦ ∷ []) "John.17.24"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.17.24"
∷ word (θ ∷ ε ∷ ω ∷ ρ ∷ ῶ ∷ σ ∷ ι ∷ ν ∷ []) "John.17.24"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.17.24"
∷ word (δ ∷ ό ∷ ξ ∷ α ∷ ν ∷ []) "John.17.24"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.17.24"
∷ word (ἐ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.17.24"
∷ word (ἣ ∷ ν ∷ []) "John.17.24"
∷ word (δ ∷ έ ∷ δ ∷ ω ∷ κ ∷ ά ∷ ς ∷ []) "John.17.24"
∷ word (μ ∷ ο ∷ ι ∷ []) "John.17.24"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.17.24"
∷ word (ἠ ∷ γ ∷ ά ∷ π ∷ η ∷ σ ∷ ά ∷ ς ∷ []) "John.17.24"
∷ word (μ ∷ ε ∷ []) "John.17.24"
∷ word (π ∷ ρ ∷ ὸ ∷ []) "John.17.24"
∷ word (κ ∷ α ∷ τ ∷ α ∷ β ∷ ο ∷ ∙λ ∷ ῆ ∷ ς ∷ []) "John.17.24"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ υ ∷ []) "John.17.24"
∷ word (Π ∷ ά ∷ τ ∷ ε ∷ ρ ∷ []) "John.17.25"
∷ word (δ ∷ ί ∷ κ ∷ α ∷ ι ∷ ε ∷ []) "John.17.25"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.17.25"
∷ word (ὁ ∷ []) "John.17.25"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ ς ∷ []) "John.17.25"
∷ word (σ ∷ ε ∷ []) "John.17.25"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.17.25"
∷ word (ἔ ∷ γ ∷ ν ∷ ω ∷ []) "John.17.25"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.17.25"
∷ word (δ ∷ έ ∷ []) "John.17.25"
∷ word (σ ∷ ε ∷ []) "John.17.25"
∷ word (ἔ ∷ γ ∷ ν ∷ ω ∷ ν ∷ []) "John.17.25"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.17.25"
∷ word (ο ∷ ὗ ∷ τ ∷ ο ∷ ι ∷ []) "John.17.25"
∷ word (ἔ ∷ γ ∷ ν ∷ ω ∷ σ ∷ α ∷ ν ∷ []) "John.17.25"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.17.25"
∷ word (σ ∷ ύ ∷ []) "John.17.25"
∷ word (μ ∷ ε ∷ []) "John.17.25"
∷ word (ἀ ∷ π ∷ έ ∷ σ ∷ τ ∷ ε ∷ ι ∷ ∙λ ∷ α ∷ ς ∷ []) "John.17.25"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.17.26"
∷ word (ἐ ∷ γ ∷ ν ∷ ώ ∷ ρ ∷ ι ∷ σ ∷ α ∷ []) "John.17.26"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.17.26"
∷ word (τ ∷ ὸ ∷ []) "John.17.26"
∷ word (ὄ ∷ ν ∷ ο ∷ μ ∷ ά ∷ []) "John.17.26"
∷ word (σ ∷ ο ∷ υ ∷ []) "John.17.26"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.17.26"
∷ word (γ ∷ ν ∷ ω ∷ ρ ∷ ί ∷ σ ∷ ω ∷ []) "John.17.26"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.17.26"
∷ word (ἡ ∷ []) "John.17.26"
∷ word (ἀ ∷ γ ∷ ά ∷ π ∷ η ∷ []) "John.17.26"
∷ word (ἣ ∷ ν ∷ []) "John.17.26"
∷ word (ἠ ∷ γ ∷ ά ∷ π ∷ η ∷ σ ∷ ά ∷ ς ∷ []) "John.17.26"
∷ word (μ ∷ ε ∷ []) "John.17.26"
∷ word (ἐ ∷ ν ∷ []) "John.17.26"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.17.26"
∷ word (ᾖ ∷ []) "John.17.26"
∷ word (κ ∷ ἀ ∷ γ ∷ ὼ ∷ []) "John.17.26"
∷ word (ἐ ∷ ν ∷ []) "John.17.26"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.17.26"
∷ word (Τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.18.1"
∷ word (ε ∷ ἰ ∷ π ∷ ὼ ∷ ν ∷ []) "John.18.1"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.18.1"
∷ word (ἐ ∷ ξ ∷ ῆ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.18.1"
∷ word (σ ∷ ὺ ∷ ν ∷ []) "John.18.1"
∷ word (τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.18.1"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ α ∷ ῖ ∷ ς ∷ []) "John.18.1"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.18.1"
∷ word (π ∷ έ ∷ ρ ∷ α ∷ ν ∷ []) "John.18.1"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.18.1"
∷ word (χ ∷ ε ∷ ι ∷ μ ∷ ά ∷ ρ ∷ ρ ∷ ο ∷ υ ∷ []) "John.18.1"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.18.1"
∷ word (Κ ∷ ε ∷ δ ∷ ρ ∷ ὼ ∷ ν ∷ []) "John.18.1"
∷ word (ὅ ∷ π ∷ ο ∷ υ ∷ []) "John.18.1"
∷ word (ἦ ∷ ν ∷ []) "John.18.1"
∷ word (κ ∷ ῆ ∷ π ∷ ο ∷ ς ∷ []) "John.18.1"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.18.1"
∷ word (ὃ ∷ ν ∷ []) "John.18.1"
∷ word (ε ∷ ἰ ∷ σ ∷ ῆ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.18.1"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ς ∷ []) "John.18.1"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.18.1"
∷ word (ο ∷ ἱ ∷ []) "John.18.1"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ α ∷ ὶ ∷ []) "John.18.1"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.18.1"
∷ word (ᾔ ∷ δ ∷ ε ∷ ι ∷ []) "John.18.2"
∷ word (δ ∷ ὲ ∷ []) "John.18.2"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.18.2"
∷ word (Ἰ ∷ ο ∷ ύ ∷ δ ∷ α ∷ ς ∷ []) "John.18.2"
∷ word (ὁ ∷ []) "John.18.2"
∷ word (π ∷ α ∷ ρ ∷ α ∷ δ ∷ ι ∷ δ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.18.2"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.18.2"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.18.2"
∷ word (τ ∷ ό ∷ π ∷ ο ∷ ν ∷ []) "John.18.2"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.18.2"
∷ word (π ∷ ο ∷ ∙λ ∷ ∙λ ∷ ά ∷ κ ∷ ι ∷ ς ∷ []) "John.18.2"
∷ word (σ ∷ υ ∷ ν ∷ ή ∷ χ ∷ θ ∷ η ∷ []) "John.18.2"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.18.2"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ []) "John.18.2"
∷ word (μ ∷ ε ∷ τ ∷ ὰ ∷ []) "John.18.2"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.18.2"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ ῶ ∷ ν ∷ []) "John.18.2"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.18.2"
∷ word (ὁ ∷ []) "John.18.3"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.18.3"
∷ word (Ἰ ∷ ο ∷ ύ ∷ δ ∷ α ∷ ς ∷ []) "John.18.3"
∷ word (∙λ ∷ α ∷ β ∷ ὼ ∷ ν ∷ []) "John.18.3"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.18.3"
∷ word (σ ∷ π ∷ ε ∷ ῖ ∷ ρ ∷ α ∷ ν ∷ []) "John.18.3"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.18.3"
∷ word (ἐ ∷ κ ∷ []) "John.18.3"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.18.3"
∷ word (ἀ ∷ ρ ∷ χ ∷ ι ∷ ε ∷ ρ ∷ έ ∷ ω ∷ ν ∷ []) "John.18.3"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.18.3"
∷ word (ἐ ∷ κ ∷ []) "John.18.3"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.18.3"
∷ word (Φ ∷ α ∷ ρ ∷ ι ∷ σ ∷ α ∷ ί ∷ ω ∷ ν ∷ []) "John.18.3"
∷ word (ὑ ∷ π ∷ η ∷ ρ ∷ έ ∷ τ ∷ α ∷ ς ∷ []) "John.18.3"
∷ word (ἔ ∷ ρ ∷ χ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.18.3"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ []) "John.18.3"
∷ word (μ ∷ ε ∷ τ ∷ ὰ ∷ []) "John.18.3"
∷ word (φ ∷ α ∷ ν ∷ ῶ ∷ ν ∷ []) "John.18.3"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.18.3"
∷ word (∙λ ∷ α ∷ μ ∷ π ∷ ά ∷ δ ∷ ω ∷ ν ∷ []) "John.18.3"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.18.3"
∷ word (ὅ ∷ π ∷ ∙λ ∷ ω ∷ ν ∷ []) "John.18.3"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.18.4"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.18.4"
∷ word (ε ∷ ἰ ∷ δ ∷ ὼ ∷ ς ∷ []) "John.18.4"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ α ∷ []) "John.18.4"
∷ word (τ ∷ ὰ ∷ []) "John.18.4"
∷ word (ἐ ∷ ρ ∷ χ ∷ ό ∷ μ ∷ ε ∷ ν ∷ α ∷ []) "John.18.4"
∷ word (ἐ ∷ π ∷ []) "John.18.4"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.18.4"
∷ word (ἐ ∷ ξ ∷ ῆ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.18.4"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.18.4"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.18.4"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.18.4"
∷ word (Τ ∷ ί ∷ ν ∷ α ∷ []) "John.18.4"
∷ word (ζ ∷ η ∷ τ ∷ ε ∷ ῖ ∷ τ ∷ ε ∷ []) "John.18.4"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.18.5"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.18.5"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ν ∷ []) "John.18.5"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.18.5"
∷ word (Ν ∷ α ∷ ζ ∷ ω ∷ ρ ∷ α ∷ ῖ ∷ ο ∷ ν ∷ []) "John.18.5"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.18.5"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.18.5"
∷ word (Ἐ ∷ γ ∷ ώ ∷ []) "John.18.5"
∷ word (ε ∷ ἰ ∷ μ ∷ ι ∷ []) "John.18.5"
∷ word (ε ∷ ἱ ∷ σ ∷ τ ∷ ή ∷ κ ∷ ε ∷ ι ∷ []) "John.18.5"
∷ word (δ ∷ ὲ ∷ []) "John.18.5"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.18.5"
∷ word (Ἰ ∷ ο ∷ ύ ∷ δ ∷ α ∷ ς ∷ []) "John.18.5"
∷ word (ὁ ∷ []) "John.18.5"
∷ word (π ∷ α ∷ ρ ∷ α ∷ δ ∷ ι ∷ δ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.18.5"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.18.5"
∷ word (μ ∷ ε ∷ τ ∷ []) "John.18.5"
∷ word (α ∷ ὐ ∷ τ ∷ ῶ ∷ ν ∷ []) "John.18.5"
∷ word (ὡ ∷ ς ∷ []) "John.18.6"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.18.6"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.18.6"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.18.6"
∷ word (Ἐ ∷ γ ∷ ώ ∷ []) "John.18.6"
∷ word (ε ∷ ἰ ∷ μ ∷ ι ∷ []) "John.18.6"
∷ word (ἀ ∷ π ∷ ῆ ∷ ∙λ ∷ θ ∷ ο ∷ ν ∷ []) "John.18.6"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.18.6"
∷ word (τ ∷ ὰ ∷ []) "John.18.6"
∷ word (ὀ ∷ π ∷ ί ∷ σ ∷ ω ∷ []) "John.18.6"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.18.6"
∷ word (ἔ ∷ π ∷ ε ∷ σ ∷ α ∷ ν ∷ []) "John.18.6"
∷ word (χ ∷ α ∷ μ ∷ α ∷ ί ∷ []) "John.18.6"
∷ word (π ∷ ά ∷ ∙λ ∷ ι ∷ ν ∷ []) "John.18.7"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.18.7"
∷ word (ἐ ∷ π ∷ η ∷ ρ ∷ ώ ∷ τ ∷ η ∷ σ ∷ ε ∷ ν ∷ []) "John.18.7"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ύ ∷ ς ∷ []) "John.18.7"
∷ word (Τ ∷ ί ∷ ν ∷ α ∷ []) "John.18.7"
∷ word (ζ ∷ η ∷ τ ∷ ε ∷ ῖ ∷ τ ∷ ε ∷ []) "John.18.7"
∷ word (ο ∷ ἱ ∷ []) "John.18.7"
∷ word (δ ∷ ὲ ∷ []) "John.18.7"
∷ word (ε ∷ ἶ ∷ π ∷ α ∷ ν ∷ []) "John.18.7"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ν ∷ []) "John.18.7"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.18.7"
∷ word (Ν ∷ α ∷ ζ ∷ ω ∷ ρ ∷ α ∷ ῖ ∷ ο ∷ ν ∷ []) "John.18.7"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.18.8"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.18.8"
∷ word (Ε ∷ ἶ ∷ π ∷ ο ∷ ν ∷ []) "John.18.8"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.18.8"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.18.8"
∷ word (ἐ ∷ γ ∷ ώ ∷ []) "John.18.8"
∷ word (ε ∷ ἰ ∷ μ ∷ ι ∷ []) "John.18.8"
∷ word (ε ∷ ἰ ∷ []) "John.18.8"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.18.8"
∷ word (ἐ ∷ μ ∷ ὲ ∷ []) "John.18.8"
∷ word (ζ ∷ η ∷ τ ∷ ε ∷ ῖ ∷ τ ∷ ε ∷ []) "John.18.8"
∷ word (ἄ ∷ φ ∷ ε ∷ τ ∷ ε ∷ []) "John.18.8"
∷ word (τ ∷ ο ∷ ύ ∷ τ ∷ ο ∷ υ ∷ ς ∷ []) "John.18.8"
∷ word (ὑ ∷ π ∷ ά ∷ γ ∷ ε ∷ ι ∷ ν ∷ []) "John.18.8"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.18.9"
∷ word (π ∷ ∙λ ∷ η ∷ ρ ∷ ω ∷ θ ∷ ῇ ∷ []) "John.18.9"
∷ word (ὁ ∷ []) "John.18.9"
∷ word (∙λ ∷ ό ∷ γ ∷ ο ∷ ς ∷ []) "John.18.9"
∷ word (ὃ ∷ ν ∷ []) "John.18.9"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.18.9"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.18.9"
∷ word (Ο ∷ ὓ ∷ ς ∷ []) "John.18.9"
∷ word (δ ∷ έ ∷ δ ∷ ω ∷ κ ∷ ά ∷ ς ∷ []) "John.18.9"
∷ word (μ ∷ ο ∷ ι ∷ []) "John.18.9"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.18.9"
∷ word (ἀ ∷ π ∷ ώ ∷ ∙λ ∷ ε ∷ σ ∷ α ∷ []) "John.18.9"
∷ word (ἐ ∷ ξ ∷ []) "John.18.9"
∷ word (α ∷ ὐ ∷ τ ∷ ῶ ∷ ν ∷ []) "John.18.9"
∷ word (ο ∷ ὐ ∷ δ ∷ έ ∷ ν ∷ α ∷ []) "John.18.9"
∷ word (Σ ∷ ί ∷ μ ∷ ω ∷ ν ∷ []) "John.18.10"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.18.10"
∷ word (Π ∷ έ ∷ τ ∷ ρ ∷ ο ∷ ς ∷ []) "John.18.10"
∷ word (ἔ ∷ χ ∷ ω ∷ ν ∷ []) "John.18.10"
∷ word (μ ∷ ά ∷ χ ∷ α ∷ ι ∷ ρ ∷ α ∷ ν ∷ []) "John.18.10"
∷ word (ε ∷ ἵ ∷ ∙λ ∷ κ ∷ υ ∷ σ ∷ ε ∷ ν ∷ []) "John.18.10"
∷ word (α ∷ ὐ ∷ τ ∷ ὴ ∷ ν ∷ []) "John.18.10"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.18.10"
∷ word (ἔ ∷ π ∷ α ∷ ι ∷ σ ∷ ε ∷ ν ∷ []) "John.18.10"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.18.10"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.18.10"
∷ word (ἀ ∷ ρ ∷ χ ∷ ι ∷ ε ∷ ρ ∷ έ ∷ ω ∷ ς ∷ []) "John.18.10"
∷ word (δ ∷ ο ∷ ῦ ∷ ∙λ ∷ ο ∷ ν ∷ []) "John.18.10"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.18.10"
∷ word (ἀ ∷ π ∷ έ ∷ κ ∷ ο ∷ ψ ∷ ε ∷ ν ∷ []) "John.18.10"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.18.10"
∷ word (τ ∷ ὸ ∷ []) "John.18.10"
∷ word (ὠ ∷ τ ∷ ά ∷ ρ ∷ ι ∷ ο ∷ ν ∷ []) "John.18.10"
∷ word (τ ∷ ὸ ∷ []) "John.18.10"
∷ word (δ ∷ ε ∷ ξ ∷ ι ∷ ό ∷ ν ∷ []) "John.18.10"
∷ word (ἦ ∷ ν ∷ []) "John.18.10"
∷ word (δ ∷ ὲ ∷ []) "John.18.10"
∷ word (ὄ ∷ ν ∷ ο ∷ μ ∷ α ∷ []) "John.18.10"
∷ word (τ ∷ ῷ ∷ []) "John.18.10"
∷ word (δ ∷ ο ∷ ύ ∷ ∙λ ∷ ῳ ∷ []) "John.18.10"
∷ word (Μ ∷ ά ∷ ∙λ ∷ χ ∷ ο ∷ ς ∷ []) "John.18.10"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.18.11"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.18.11"
∷ word (ὁ ∷ []) "John.18.11"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.18.11"
∷ word (τ ∷ ῷ ∷ []) "John.18.11"
∷ word (Π ∷ έ ∷ τ ∷ ρ ∷ ῳ ∷ []) "John.18.11"
∷ word (Β ∷ ά ∷ ∙λ ∷ ε ∷ []) "John.18.11"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.18.11"
∷ word (μ ∷ ά ∷ χ ∷ α ∷ ι ∷ ρ ∷ α ∷ ν ∷ []) "John.18.11"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.18.11"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.18.11"
∷ word (θ ∷ ή ∷ κ ∷ η ∷ ν ∷ []) "John.18.11"
∷ word (τ ∷ ὸ ∷ []) "John.18.11"
∷ word (π ∷ ο ∷ τ ∷ ή ∷ ρ ∷ ι ∷ ο ∷ ν ∷ []) "John.18.11"
∷ word (ὃ ∷ []) "John.18.11"
∷ word (δ ∷ έ ∷ δ ∷ ω ∷ κ ∷ έ ∷ ν ∷ []) "John.18.11"
∷ word (μ ∷ ο ∷ ι ∷ []) "John.18.11"
∷ word (ὁ ∷ []) "John.18.11"
∷ word (π ∷ α ∷ τ ∷ ὴ ∷ ρ ∷ []) "John.18.11"
∷ word (ο ∷ ὐ ∷ []) "John.18.11"
∷ word (μ ∷ ὴ ∷ []) "John.18.11"
∷ word (π ∷ ί ∷ ω ∷ []) "John.18.11"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ []) "John.18.11"
∷ word (Ἡ ∷ []) "John.18.12"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.18.12"
∷ word (σ ∷ π ∷ ε ∷ ῖ ∷ ρ ∷ α ∷ []) "John.18.12"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.18.12"
∷ word (ὁ ∷ []) "John.18.12"
∷ word (χ ∷ ι ∷ ∙λ ∷ ί ∷ α ∷ ρ ∷ χ ∷ ο ∷ ς ∷ []) "John.18.12"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.18.12"
∷ word (ο ∷ ἱ ∷ []) "John.18.12"
∷ word (ὑ ∷ π ∷ η ∷ ρ ∷ έ ∷ τ ∷ α ∷ ι ∷ []) "John.18.12"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.18.12"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ί ∷ ω ∷ ν ∷ []) "John.18.12"
∷ word (σ ∷ υ ∷ ν ∷ έ ∷ ∙λ ∷ α ∷ β ∷ ο ∷ ν ∷ []) "John.18.12"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.18.12"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ν ∷ []) "John.18.12"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.18.12"
∷ word (ἔ ∷ δ ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.18.12"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.18.12"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.18.13"
∷ word (ἤ ∷ γ ∷ α ∷ γ ∷ ο ∷ ν ∷ []) "John.18.13"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.18.13"
∷ word (Ἅ ∷ ν ∷ ν ∷ α ∷ ν ∷ []) "John.18.13"
∷ word (π ∷ ρ ∷ ῶ ∷ τ ∷ ο ∷ ν ∷ []) "John.18.13"
∷ word (ἦ ∷ ν ∷ []) "John.18.13"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.18.13"
∷ word (π ∷ ε ∷ ν ∷ θ ∷ ε ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.18.13"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.18.13"
∷ word (Κ ∷ α ∷ ϊ ∷ ά ∷ φ ∷ α ∷ []) "John.18.13"
∷ word (ὃ ∷ ς ∷ []) "John.18.13"
∷ word (ἦ ∷ ν ∷ []) "John.18.13"
∷ word (ἀ ∷ ρ ∷ χ ∷ ι ∷ ε ∷ ρ ∷ ε ∷ ὺ ∷ ς ∷ []) "John.18.13"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.18.13"
∷ word (ἐ ∷ ν ∷ ι ∷ α ∷ υ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.18.13"
∷ word (ἐ ∷ κ ∷ ε ∷ ί ∷ ν ∷ ο ∷ υ ∷ []) "John.18.13"
∷ word (ἦ ∷ ν ∷ []) "John.18.14"
∷ word (δ ∷ ὲ ∷ []) "John.18.14"
∷ word (Κ ∷ α ∷ ϊ ∷ ά ∷ φ ∷ α ∷ ς ∷ []) "John.18.14"
∷ word (ὁ ∷ []) "John.18.14"
∷ word (σ ∷ υ ∷ μ ∷ β ∷ ο ∷ υ ∷ ∙λ ∷ ε ∷ ύ ∷ σ ∷ α ∷ ς ∷ []) "John.18.14"
∷ word (τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.18.14"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ί ∷ ο ∷ ι ∷ ς ∷ []) "John.18.14"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.18.14"
∷ word (σ ∷ υ ∷ μ ∷ φ ∷ έ ∷ ρ ∷ ε ∷ ι ∷ []) "John.18.14"
∷ word (ἕ ∷ ν ∷ α ∷ []) "John.18.14"
∷ word (ἄ ∷ ν ∷ θ ∷ ρ ∷ ω ∷ π ∷ ο ∷ ν ∷ []) "John.18.14"
∷ word (ἀ ∷ π ∷ ο ∷ θ ∷ α ∷ ν ∷ ε ∷ ῖ ∷ ν ∷ []) "John.18.14"
∷ word (ὑ ∷ π ∷ ὲ ∷ ρ ∷ []) "John.18.14"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.18.14"
∷ word (∙λ ∷ α ∷ ο ∷ ῦ ∷ []) "John.18.14"
∷ word (Ἠ ∷ κ ∷ ο ∷ ∙λ ∷ ο ∷ ύ ∷ θ ∷ ε ∷ ι ∷ []) "John.18.15"
∷ word (δ ∷ ὲ ∷ []) "John.18.15"
∷ word (τ ∷ ῷ ∷ []) "John.18.15"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ []) "John.18.15"
∷ word (Σ ∷ ί ∷ μ ∷ ω ∷ ν ∷ []) "John.18.15"
∷ word (Π ∷ έ ∷ τ ∷ ρ ∷ ο ∷ ς ∷ []) "John.18.15"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.18.15"
∷ word (ἄ ∷ ∙λ ∷ ∙λ ∷ ο ∷ ς ∷ []) "John.18.15"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ ή ∷ ς ∷ []) "John.18.15"
∷ word (ὁ ∷ []) "John.18.15"
∷ word (δ ∷ ὲ ∷ []) "John.18.15"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ ὴ ∷ ς ∷ []) "John.18.15"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ο ∷ ς ∷ []) "John.18.15"
∷ word (ἦ ∷ ν ∷ []) "John.18.15"
∷ word (γ ∷ ν ∷ ω ∷ σ ∷ τ ∷ ὸ ∷ ς ∷ []) "John.18.15"
∷ word (τ ∷ ῷ ∷ []) "John.18.15"
∷ word (ἀ ∷ ρ ∷ χ ∷ ι ∷ ε ∷ ρ ∷ ε ∷ ῖ ∷ []) "John.18.15"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.18.15"
∷ word (σ ∷ υ ∷ ν ∷ ε ∷ ι ∷ σ ∷ ῆ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.18.15"
∷ word (τ ∷ ῷ ∷ []) "John.18.15"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ []) "John.18.15"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.18.15"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.18.15"
∷ word (α ∷ ὐ ∷ ∙λ ∷ ὴ ∷ ν ∷ []) "John.18.15"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.18.15"
∷ word (ἀ ∷ ρ ∷ χ ∷ ι ∷ ε ∷ ρ ∷ έ ∷ ω ∷ ς ∷ []) "John.18.15"
∷ word (ὁ ∷ []) "John.18.16"
∷ word (δ ∷ ὲ ∷ []) "John.18.16"
∷ word (Π ∷ έ ∷ τ ∷ ρ ∷ ο ∷ ς ∷ []) "John.18.16"
∷ word (ε ∷ ἱ ∷ σ ∷ τ ∷ ή ∷ κ ∷ ε ∷ ι ∷ []) "John.18.16"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.18.16"
∷ word (τ ∷ ῇ ∷ []) "John.18.16"
∷ word (θ ∷ ύ ∷ ρ ∷ ᾳ ∷ []) "John.18.16"
∷ word (ἔ ∷ ξ ∷ ω ∷ []) "John.18.16"
∷ word (ἐ ∷ ξ ∷ ῆ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.18.16"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.18.16"
∷ word (ὁ ∷ []) "John.18.16"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ ὴ ∷ ς ∷ []) "John.18.16"
∷ word (ὁ ∷ []) "John.18.16"
∷ word (ἄ ∷ ∙λ ∷ ∙λ ∷ ο ∷ ς ∷ []) "John.18.16"
∷ word (ὁ ∷ []) "John.18.16"
∷ word (γ ∷ ν ∷ ω ∷ σ ∷ τ ∷ ὸ ∷ ς ∷ []) "John.18.16"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.18.16"
∷ word (ἀ ∷ ρ ∷ χ ∷ ι ∷ ε ∷ ρ ∷ έ ∷ ω ∷ ς ∷ []) "John.18.16"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.18.16"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.18.16"
∷ word (τ ∷ ῇ ∷ []) "John.18.16"
∷ word (θ ∷ υ ∷ ρ ∷ ω ∷ ρ ∷ ῷ ∷ []) "John.18.16"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.18.16"
∷ word (ε ∷ ἰ ∷ σ ∷ ή ∷ γ ∷ α ∷ γ ∷ ε ∷ ν ∷ []) "John.18.16"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.18.16"
∷ word (Π ∷ έ ∷ τ ∷ ρ ∷ ο ∷ ν ∷ []) "John.18.16"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.18.17"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.18.17"
∷ word (τ ∷ ῷ ∷ []) "John.18.17"
∷ word (Π ∷ έ ∷ τ ∷ ρ ∷ ῳ ∷ []) "John.18.17"
∷ word (ἡ ∷ []) "John.18.17"
∷ word (π ∷ α ∷ ι ∷ δ ∷ ί ∷ σ ∷ κ ∷ η ∷ []) "John.18.17"
∷ word (ἡ ∷ []) "John.18.17"
∷ word (θ ∷ υ ∷ ρ ∷ ω ∷ ρ ∷ ό ∷ ς ∷ []) "John.18.17"
∷ word (Μ ∷ ὴ ∷ []) "John.18.17"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.18.17"
∷ word (σ ∷ ὺ ∷ []) "John.18.17"
∷ word (ἐ ∷ κ ∷ []) "John.18.17"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.18.17"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ ῶ ∷ ν ∷ []) "John.18.17"
∷ word (ε ∷ ἶ ∷ []) "John.18.17"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.18.17"
∷ word (ἀ ∷ ν ∷ θ ∷ ρ ∷ ώ ∷ π ∷ ο ∷ υ ∷ []) "John.18.17"
∷ word (τ ∷ ο ∷ ύ ∷ τ ∷ ο ∷ υ ∷ []) "John.18.17"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.18.17"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ο ∷ ς ∷ []) "John.18.17"
∷ word (Ο ∷ ὐ ∷ κ ∷ []) "John.18.17"
∷ word (ε ∷ ἰ ∷ μ ∷ ί ∷ []) "John.18.17"
∷ word (ε ∷ ἱ ∷ σ ∷ τ ∷ ή ∷ κ ∷ ε ∷ ι ∷ σ ∷ α ∷ ν ∷ []) "John.18.18"
∷ word (δ ∷ ὲ ∷ []) "John.18.18"
∷ word (ο ∷ ἱ ∷ []) "John.18.18"
∷ word (δ ∷ ο ∷ ῦ ∷ ∙λ ∷ ο ∷ ι ∷ []) "John.18.18"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.18.18"
∷ word (ο ∷ ἱ ∷ []) "John.18.18"
∷ word (ὑ ∷ π ∷ η ∷ ρ ∷ έ ∷ τ ∷ α ∷ ι ∷ []) "John.18.18"
∷ word (ἀ ∷ ν ∷ θ ∷ ρ ∷ α ∷ κ ∷ ι ∷ ὰ ∷ ν ∷ []) "John.18.18"
∷ word (π ∷ ε ∷ π ∷ ο ∷ ι ∷ η ∷ κ ∷ ό ∷ τ ∷ ε ∷ ς ∷ []) "John.18.18"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.18.18"
∷ word (ψ ∷ ῦ ∷ χ ∷ ο ∷ ς ∷ []) "John.18.18"
∷ word (ἦ ∷ ν ∷ []) "John.18.18"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.18.18"
∷ word (ἐ ∷ θ ∷ ε ∷ ρ ∷ μ ∷ α ∷ ί ∷ ν ∷ ο ∷ ν ∷ τ ∷ ο ∷ []) "John.18.18"
∷ word (ἦ ∷ ν ∷ []) "John.18.18"
∷ word (δ ∷ ὲ ∷ []) "John.18.18"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.18.18"
∷ word (ὁ ∷ []) "John.18.18"
∷ word (Π ∷ έ ∷ τ ∷ ρ ∷ ο ∷ ς ∷ []) "John.18.18"
∷ word (μ ∷ ε ∷ τ ∷ []) "John.18.18"
∷ word (α ∷ ὐ ∷ τ ∷ ῶ ∷ ν ∷ []) "John.18.18"
∷ word (ἑ ∷ σ ∷ τ ∷ ὼ ∷ ς ∷ []) "John.18.18"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.18.18"
∷ word (θ ∷ ε ∷ ρ ∷ μ ∷ α ∷ ι ∷ ν ∷ ό ∷ μ ∷ ε ∷ ν ∷ ο ∷ ς ∷ []) "John.18.18"
∷ word (Ὁ ∷ []) "John.18.19"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.18.19"
∷ word (ἀ ∷ ρ ∷ χ ∷ ι ∷ ε ∷ ρ ∷ ε ∷ ὺ ∷ ς ∷ []) "John.18.19"
∷ word (ἠ ∷ ρ ∷ ώ ∷ τ ∷ η ∷ σ ∷ ε ∷ ν ∷ []) "John.18.19"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.18.19"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ν ∷ []) "John.18.19"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.18.19"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.18.19"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ ῶ ∷ ν ∷ []) "John.18.19"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.18.19"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.18.19"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.18.19"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.18.19"
∷ word (δ ∷ ι ∷ δ ∷ α ∷ χ ∷ ῆ ∷ ς ∷ []) "John.18.19"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.18.19"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.18.20"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.18.20"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.18.20"
∷ word (Ἐ ∷ γ ∷ ὼ ∷ []) "John.18.20"
∷ word (π ∷ α ∷ ρ ∷ ρ ∷ η ∷ σ ∷ ί ∷ ᾳ ∷ []) "John.18.20"
∷ word (∙λ ∷ ε ∷ ∙λ ∷ ά ∷ ∙λ ∷ η ∷ κ ∷ α ∷ []) "John.18.20"
∷ word (τ ∷ ῷ ∷ []) "John.18.20"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ῳ ∷ []) "John.18.20"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.18.20"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ ο ∷ τ ∷ ε ∷ []) "John.18.20"
∷ word (ἐ ∷ δ ∷ ί ∷ δ ∷ α ∷ ξ ∷ α ∷ []) "John.18.20"
∷ word (ἐ ∷ ν ∷ []) "John.18.20"
∷ word (σ ∷ υ ∷ ν ∷ α ∷ γ ∷ ω ∷ γ ∷ ῇ ∷ []) "John.18.20"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.18.20"
∷ word (ἐ ∷ ν ∷ []) "John.18.20"
∷ word (τ ∷ ῷ ∷ []) "John.18.20"
∷ word (ἱ ∷ ε ∷ ρ ∷ ῷ ∷ []) "John.18.20"
∷ word (ὅ ∷ π ∷ ο ∷ υ ∷ []) "John.18.20"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.18.20"
∷ word (ο ∷ ἱ ∷ []) "John.18.20"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ῖ ∷ ο ∷ ι ∷ []) "John.18.20"
∷ word (σ ∷ υ ∷ ν ∷ έ ∷ ρ ∷ χ ∷ ο ∷ ν ∷ τ ∷ α ∷ ι ∷ []) "John.18.20"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.18.20"
∷ word (ἐ ∷ ν ∷ []) "John.18.20"
∷ word (κ ∷ ρ ∷ υ ∷ π ∷ τ ∷ ῷ ∷ []) "John.18.20"
∷ word (ἐ ∷ ∙λ ∷ ά ∷ ∙λ ∷ η ∷ σ ∷ α ∷ []) "John.18.20"
∷ word (ο ∷ ὐ ∷ δ ∷ έ ∷ ν ∷ []) "John.18.20"
∷ word (τ ∷ ί ∷ []) "John.18.21"
∷ word (μ ∷ ε ∷ []) "John.18.21"
∷ word (ἐ ∷ ρ ∷ ω ∷ τ ∷ ᾷ ∷ ς ∷ []) "John.18.21"
∷ word (ἐ ∷ ρ ∷ ώ ∷ τ ∷ η ∷ σ ∷ ο ∷ ν ∷ []) "John.18.21"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.18.21"
∷ word (ἀ ∷ κ ∷ η ∷ κ ∷ ο ∷ ό ∷ τ ∷ α ∷ ς ∷ []) "John.18.21"
∷ word (τ ∷ ί ∷ []) "John.18.21"
∷ word (ἐ ∷ ∙λ ∷ ά ∷ ∙λ ∷ η ∷ σ ∷ α ∷ []) "John.18.21"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.18.21"
∷ word (ἴ ∷ δ ∷ ε ∷ []) "John.18.21"
∷ word (ο ∷ ὗ ∷ τ ∷ ο ∷ ι ∷ []) "John.18.21"
∷ word (ο ∷ ἴ ∷ δ ∷ α ∷ σ ∷ ι ∷ ν ∷ []) "John.18.21"
∷ word (ἃ ∷ []) "John.18.21"
∷ word (ε ∷ ἶ ∷ π ∷ ο ∷ ν ∷ []) "John.18.21"
∷ word (ἐ ∷ γ ∷ ώ ∷ []) "John.18.21"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.18.22"
∷ word (δ ∷ ὲ ∷ []) "John.18.22"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.18.22"
∷ word (ε ∷ ἰ ∷ π ∷ ό ∷ ν ∷ τ ∷ ο ∷ ς ∷ []) "John.18.22"
∷ word (ε ∷ ἷ ∷ ς ∷ []) "John.18.22"
∷ word (π ∷ α ∷ ρ ∷ ε ∷ σ ∷ τ ∷ η ∷ κ ∷ ὼ ∷ ς ∷ []) "John.18.22"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.18.22"
∷ word (ὑ ∷ π ∷ η ∷ ρ ∷ ε ∷ τ ∷ ῶ ∷ ν ∷ []) "John.18.22"
∷ word (ἔ ∷ δ ∷ ω ∷ κ ∷ ε ∷ ν ∷ []) "John.18.22"
∷ word (ῥ ∷ ά ∷ π ∷ ι ∷ σ ∷ μ ∷ α ∷ []) "John.18.22"
∷ word (τ ∷ ῷ ∷ []) "John.18.22"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ []) "John.18.22"
∷ word (ε ∷ ἰ ∷ π ∷ ώ ∷ ν ∷ []) "John.18.22"
∷ word (Ο ∷ ὕ ∷ τ ∷ ω ∷ ς ∷ []) "John.18.22"
∷ word (ἀ ∷ π ∷ ο ∷ κ ∷ ρ ∷ ί ∷ ν ∷ ῃ ∷ []) "John.18.22"
∷ word (τ ∷ ῷ ∷ []) "John.18.22"
∷ word (ἀ ∷ ρ ∷ χ ∷ ι ∷ ε ∷ ρ ∷ ε ∷ ῖ ∷ []) "John.18.22"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.18.23"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.18.23"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.18.23"
∷ word (Ε ∷ ἰ ∷ []) "John.18.23"
∷ word (κ ∷ α ∷ κ ∷ ῶ ∷ ς ∷ []) "John.18.23"
∷ word (ἐ ∷ ∙λ ∷ ά ∷ ∙λ ∷ η ∷ σ ∷ α ∷ []) "John.18.23"
∷ word (μ ∷ α ∷ ρ ∷ τ ∷ ύ ∷ ρ ∷ η ∷ σ ∷ ο ∷ ν ∷ []) "John.18.23"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.18.23"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.18.23"
∷ word (κ ∷ α ∷ κ ∷ ο ∷ ῦ ∷ []) "John.18.23"
∷ word (ε ∷ ἰ ∷ []) "John.18.23"
∷ word (δ ∷ ὲ ∷ []) "John.18.23"
∷ word (κ ∷ α ∷ ∙λ ∷ ῶ ∷ ς ∷ []) "John.18.23"
∷ word (τ ∷ ί ∷ []) "John.18.23"
∷ word (μ ∷ ε ∷ []) "John.18.23"
∷ word (δ ∷ έ ∷ ρ ∷ ε ∷ ι ∷ ς ∷ []) "John.18.23"
∷ word (ἀ ∷ π ∷ έ ∷ σ ∷ τ ∷ ε ∷ ι ∷ ∙λ ∷ ε ∷ ν ∷ []) "John.18.24"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.18.24"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.18.24"
∷ word (ὁ ∷ []) "John.18.24"
∷ word (Ἅ ∷ ν ∷ ν ∷ α ∷ ς ∷ []) "John.18.24"
∷ word (δ ∷ ε ∷ δ ∷ ε ∷ μ ∷ έ ∷ ν ∷ ο ∷ ν ∷ []) "John.18.24"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.18.24"
∷ word (Κ ∷ α ∷ ϊ ∷ ά ∷ φ ∷ α ∷ ν ∷ []) "John.18.24"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.18.24"
∷ word (ἀ ∷ ρ ∷ χ ∷ ι ∷ ε ∷ ρ ∷ έ ∷ α ∷ []) "John.18.24"
∷ word (Ἦ ∷ ν ∷ []) "John.18.25"
∷ word (δ ∷ ὲ ∷ []) "John.18.25"
∷ word (Σ ∷ ί ∷ μ ∷ ω ∷ ν ∷ []) "John.18.25"
∷ word (Π ∷ έ ∷ τ ∷ ρ ∷ ο ∷ ς ∷ []) "John.18.25"
∷ word (ἑ ∷ σ ∷ τ ∷ ὼ ∷ ς ∷ []) "John.18.25"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.18.25"
∷ word (θ ∷ ε ∷ ρ ∷ μ ∷ α ∷ ι ∷ ν ∷ ό ∷ μ ∷ ε ∷ ν ∷ ο ∷ ς ∷ []) "John.18.25"
∷ word (ε ∷ ἶ ∷ π ∷ ο ∷ ν ∷ []) "John.18.25"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.18.25"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.18.25"
∷ word (Μ ∷ ὴ ∷ []) "John.18.25"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.18.25"
∷ word (σ ∷ ὺ ∷ []) "John.18.25"
∷ word (ἐ ∷ κ ∷ []) "John.18.25"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.18.25"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ ῶ ∷ ν ∷ []) "John.18.25"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.18.25"
∷ word (ε ∷ ἶ ∷ []) "John.18.25"
∷ word (ἠ ∷ ρ ∷ ν ∷ ή ∷ σ ∷ α ∷ τ ∷ ο ∷ []) "John.18.25"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ο ∷ ς ∷ []) "John.18.25"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.18.25"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.18.25"
∷ word (Ο ∷ ὐ ∷ κ ∷ []) "John.18.25"
∷ word (ε ∷ ἰ ∷ μ ∷ ί ∷ []) "John.18.25"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.18.26"
∷ word (ε ∷ ἷ ∷ ς ∷ []) "John.18.26"
∷ word (ἐ ∷ κ ∷ []) "John.18.26"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.18.26"
∷ word (δ ∷ ο ∷ ύ ∷ ∙λ ∷ ω ∷ ν ∷ []) "John.18.26"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.18.26"
∷ word (ἀ ∷ ρ ∷ χ ∷ ι ∷ ε ∷ ρ ∷ έ ∷ ω ∷ ς ∷ []) "John.18.26"
∷ word (σ ∷ υ ∷ γ ∷ γ ∷ ε ∷ ν ∷ ὴ ∷ ς ∷ []) "John.18.26"
∷ word (ὢ ∷ ν ∷ []) "John.18.26"
∷ word (ο ∷ ὗ ∷ []) "John.18.26"
∷ word (ἀ ∷ π ∷ έ ∷ κ ∷ ο ∷ ψ ∷ ε ∷ ν ∷ []) "John.18.26"
∷ word (Π ∷ έ ∷ τ ∷ ρ ∷ ο ∷ ς ∷ []) "John.18.26"
∷ word (τ ∷ ὸ ∷ []) "John.18.26"
∷ word (ὠ ∷ τ ∷ ί ∷ ο ∷ ν ∷ []) "John.18.26"
∷ word (Ο ∷ ὐ ∷ κ ∷ []) "John.18.26"
∷ word (ἐ ∷ γ ∷ ώ ∷ []) "John.18.26"
∷ word (σ ∷ ε ∷ []) "John.18.26"
∷ word (ε ∷ ἶ ∷ δ ∷ ο ∷ ν ∷ []) "John.18.26"
∷ word (ἐ ∷ ν ∷ []) "John.18.26"
∷ word (τ ∷ ῷ ∷ []) "John.18.26"
∷ word (κ ∷ ή ∷ π ∷ ῳ ∷ []) "John.18.26"
∷ word (μ ∷ ε ∷ τ ∷ []) "John.18.26"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.18.26"
∷ word (π ∷ ά ∷ ∙λ ∷ ι ∷ ν ∷ []) "John.18.27"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.18.27"
∷ word (ἠ ∷ ρ ∷ ν ∷ ή ∷ σ ∷ α ∷ τ ∷ ο ∷ []) "John.18.27"
∷ word (Π ∷ έ ∷ τ ∷ ρ ∷ ο ∷ ς ∷ []) "John.18.27"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.18.27"
∷ word (ε ∷ ὐ ∷ θ ∷ έ ∷ ω ∷ ς ∷ []) "John.18.27"
∷ word (ἀ ∷ ∙λ ∷ έ ∷ κ ∷ τ ∷ ω ∷ ρ ∷ []) "John.18.27"
∷ word (ἐ ∷ φ ∷ ώ ∷ ν ∷ η ∷ σ ∷ ε ∷ ν ∷ []) "John.18.27"
∷ word (Ἄ ∷ γ ∷ ο ∷ υ ∷ σ ∷ ι ∷ ν ∷ []) "John.18.28"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.18.28"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.18.28"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ν ∷ []) "John.18.28"
∷ word (ἀ ∷ π ∷ ὸ ∷ []) "John.18.28"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.18.28"
∷ word (Κ ∷ α ∷ ϊ ∷ ά ∷ φ ∷ α ∷ []) "John.18.28"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.18.28"
∷ word (τ ∷ ὸ ∷ []) "John.18.28"
∷ word (π ∷ ρ ∷ α ∷ ι ∷ τ ∷ ώ ∷ ρ ∷ ι ∷ ο ∷ ν ∷ []) "John.18.28"
∷ word (ἦ ∷ ν ∷ []) "John.18.28"
∷ word (δ ∷ ὲ ∷ []) "John.18.28"
∷ word (π ∷ ρ ∷ ω ∷ ΐ ∷ []) "John.18.28"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.18.28"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ὶ ∷ []) "John.18.28"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.18.28"
∷ word (ε ∷ ἰ ∷ σ ∷ ῆ ∷ ∙λ ∷ θ ∷ ο ∷ ν ∷ []) "John.18.28"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.18.28"
∷ word (τ ∷ ὸ ∷ []) "John.18.28"
∷ word (π ∷ ρ ∷ α ∷ ι ∷ τ ∷ ώ ∷ ρ ∷ ι ∷ ο ∷ ν ∷ []) "John.18.28"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.18.28"
∷ word (μ ∷ ὴ ∷ []) "John.18.28"
∷ word (μ ∷ ι ∷ α ∷ ν ∷ θ ∷ ῶ ∷ σ ∷ ι ∷ ν ∷ []) "John.18.28"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.18.28"
∷ word (φ ∷ ά ∷ γ ∷ ω ∷ σ ∷ ι ∷ ν ∷ []) "John.18.28"
∷ word (τ ∷ ὸ ∷ []) "John.18.28"
∷ word (π ∷ ά ∷ σ ∷ χ ∷ α ∷ []) "John.18.28"
∷ word (ἐ ∷ ξ ∷ ῆ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.18.29"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.18.29"
∷ word (ὁ ∷ []) "John.18.29"
∷ word (Π ∷ ι ∷ ∙λ ∷ ᾶ ∷ τ ∷ ο ∷ ς ∷ []) "John.18.29"
∷ word (ἔ ∷ ξ ∷ ω ∷ []) "John.18.29"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.18.29"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.18.29"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.18.29"
∷ word (φ ∷ η ∷ σ ∷ ί ∷ ν ∷ []) "John.18.29"
∷ word (Τ ∷ ί ∷ ν ∷ α ∷ []) "John.18.29"
∷ word (κ ∷ α ∷ τ ∷ η ∷ γ ∷ ο ∷ ρ ∷ ί ∷ α ∷ ν ∷ []) "John.18.29"
∷ word (φ ∷ έ ∷ ρ ∷ ε ∷ τ ∷ ε ∷ []) "John.18.29"
∷ word (κ ∷ α ∷ τ ∷ ὰ ∷ []) "John.18.29"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.18.29"
∷ word (ἀ ∷ ν ∷ θ ∷ ρ ∷ ώ ∷ π ∷ ο ∷ υ ∷ []) "John.18.29"
∷ word (τ ∷ ο ∷ ύ ∷ τ ∷ ο ∷ υ ∷ []) "John.18.29"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.18.30"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.18.30"
∷ word (ε ∷ ἶ ∷ π ∷ α ∷ ν ∷ []) "John.18.30"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.18.30"
∷ word (Ε ∷ ἰ ∷ []) "John.18.30"
∷ word (μ ∷ ὴ ∷ []) "John.18.30"
∷ word (ἦ ∷ ν ∷ []) "John.18.30"
∷ word (ο ∷ ὗ ∷ τ ∷ ο ∷ ς ∷ []) "John.18.30"
∷ word (κ ∷ α ∷ κ ∷ ὸ ∷ ν ∷ []) "John.18.30"
∷ word (π ∷ ο ∷ ι ∷ ῶ ∷ ν ∷ []) "John.18.30"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.18.30"
∷ word (ἄ ∷ ν ∷ []) "John.18.30"
∷ word (σ ∷ ο ∷ ι ∷ []) "John.18.30"
∷ word (π ∷ α ∷ ρ ∷ ε ∷ δ ∷ ώ ∷ κ ∷ α ∷ μ ∷ ε ∷ ν ∷ []) "John.18.30"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.18.30"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.18.31"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.18.31"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.18.31"
∷ word (ὁ ∷ []) "John.18.31"
∷ word (Π ∷ ι ∷ ∙λ ∷ ᾶ ∷ τ ∷ ο ∷ ς ∷ []) "John.18.31"
∷ word (Λ ∷ ά ∷ β ∷ ε ∷ τ ∷ ε ∷ []) "John.18.31"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.18.31"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.18.31"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.18.31"
∷ word (κ ∷ α ∷ τ ∷ ὰ ∷ []) "John.18.31"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.18.31"
∷ word (ν ∷ ό ∷ μ ∷ ο ∷ ν ∷ []) "John.18.31"
∷ word (ὑ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.18.31"
∷ word (κ ∷ ρ ∷ ί ∷ ν ∷ α ∷ τ ∷ ε ∷ []) "John.18.31"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.18.31"
∷ word (ε ∷ ἶ ∷ π ∷ ο ∷ ν ∷ []) "John.18.31"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.18.31"
∷ word (ο ∷ ἱ ∷ []) "John.18.31"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ῖ ∷ ο ∷ ι ∷ []) "John.18.31"
∷ word (Ἡ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.18.31"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.18.31"
∷ word (ἔ ∷ ξ ∷ ε ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.18.31"
∷ word (ἀ ∷ π ∷ ο ∷ κ ∷ τ ∷ ε ∷ ῖ ∷ ν ∷ α ∷ ι ∷ []) "John.18.31"
∷ word (ο ∷ ὐ ∷ δ ∷ έ ∷ ν ∷ α ∷ []) "John.18.31"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.18.32"
∷ word (ὁ ∷ []) "John.18.32"
∷ word (∙λ ∷ ό ∷ γ ∷ ο ∷ ς ∷ []) "John.18.32"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.18.32"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ []) "John.18.32"
∷ word (π ∷ ∙λ ∷ η ∷ ρ ∷ ω ∷ θ ∷ ῇ ∷ []) "John.18.32"
∷ word (ὃ ∷ ν ∷ []) "John.18.32"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.18.32"
∷ word (σ ∷ η ∷ μ ∷ α ∷ ί ∷ ν ∷ ω ∷ ν ∷ []) "John.18.32"
∷ word (π ∷ ο ∷ ί ∷ ῳ ∷ []) "John.18.32"
∷ word (θ ∷ α ∷ ν ∷ ά ∷ τ ∷ ῳ ∷ []) "John.18.32"
∷ word (ἤ ∷ μ ∷ ε ∷ ∙λ ∷ ∙λ ∷ ε ∷ ν ∷ []) "John.18.32"
∷ word (ἀ ∷ π ∷ ο ∷ θ ∷ ν ∷ ῄ ∷ σ ∷ κ ∷ ε ∷ ι ∷ ν ∷ []) "John.18.32"
∷ word (Ε ∷ ἰ ∷ σ ∷ ῆ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.18.33"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.18.33"
∷ word (π ∷ ά ∷ ∙λ ∷ ι ∷ ν ∷ []) "John.18.33"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.18.33"
∷ word (τ ∷ ὸ ∷ []) "John.18.33"
∷ word (π ∷ ρ ∷ α ∷ ι ∷ τ ∷ ώ ∷ ρ ∷ ι ∷ ο ∷ ν ∷ []) "John.18.33"
∷ word (ὁ ∷ []) "John.18.33"
∷ word (Π ∷ ι ∷ ∙λ ∷ ᾶ ∷ τ ∷ ο ∷ ς ∷ []) "John.18.33"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.18.33"
∷ word (ἐ ∷ φ ∷ ώ ∷ ν ∷ η ∷ σ ∷ ε ∷ ν ∷ []) "John.18.33"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.18.33"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ν ∷ []) "John.18.33"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.18.33"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.18.33"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.18.33"
∷ word (Σ ∷ ὺ ∷ []) "John.18.33"
∷ word (ε ∷ ἶ ∷ []) "John.18.33"
∷ word (ὁ ∷ []) "John.18.33"
∷ word (β ∷ α ∷ σ ∷ ι ∷ ∙λ ∷ ε ∷ ὺ ∷ ς ∷ []) "John.18.33"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.18.33"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ί ∷ ω ∷ ν ∷ []) "John.18.33"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.18.34"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.18.34"
∷ word (Ἀ ∷ π ∷ ὸ ∷ []) "John.18.34"
∷ word (σ ∷ ε ∷ α ∷ υ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.18.34"
∷ word (σ ∷ ὺ ∷ []) "John.18.34"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.18.34"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ ς ∷ []) "John.18.34"
∷ word (ἢ ∷ []) "John.18.34"
∷ word (ἄ ∷ ∙λ ∷ ∙λ ∷ ο ∷ ι ∷ []) "John.18.34"
∷ word (ε ∷ ἶ ∷ π ∷ ό ∷ ν ∷ []) "John.18.34"
∷ word (σ ∷ ο ∷ ι ∷ []) "John.18.34"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.18.34"
∷ word (ἐ ∷ μ ∷ ο ∷ ῦ ∷ []) "John.18.34"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.18.35"
∷ word (ὁ ∷ []) "John.18.35"
∷ word (Π ∷ ι ∷ ∙λ ∷ ᾶ ∷ τ ∷ ο ∷ ς ∷ []) "John.18.35"
∷ word (Μ ∷ ή ∷ τ ∷ ι ∷ []) "John.18.35"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.18.35"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ῖ ∷ ό ∷ ς ∷ []) "John.18.35"
∷ word (ε ∷ ἰ ∷ μ ∷ ι ∷ []) "John.18.35"
∷ word (τ ∷ ὸ ∷ []) "John.18.35"
∷ word (ἔ ∷ θ ∷ ν ∷ ο ∷ ς ∷ []) "John.18.35"
∷ word (τ ∷ ὸ ∷ []) "John.18.35"
∷ word (σ ∷ ὸ ∷ ν ∷ []) "John.18.35"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.18.35"
∷ word (ο ∷ ἱ ∷ []) "John.18.35"
∷ word (ἀ ∷ ρ ∷ χ ∷ ι ∷ ε ∷ ρ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.18.35"
∷ word (π ∷ α ∷ ρ ∷ έ ∷ δ ∷ ω ∷ κ ∷ ά ∷ ν ∷ []) "John.18.35"
∷ word (σ ∷ ε ∷ []) "John.18.35"
∷ word (ἐ ∷ μ ∷ ο ∷ ί ∷ []) "John.18.35"
∷ word (τ ∷ ί ∷ []) "John.18.35"
∷ word (ἐ ∷ π ∷ ο ∷ ί ∷ η ∷ σ ∷ α ∷ ς ∷ []) "John.18.35"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.18.36"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.18.36"
∷ word (Ἡ ∷ []) "John.18.36"
∷ word (β ∷ α ∷ σ ∷ ι ∷ ∙λ ∷ ε ∷ ί ∷ α ∷ []) "John.18.36"
∷ word (ἡ ∷ []) "John.18.36"
∷ word (ἐ ∷ μ ∷ ὴ ∷ []) "John.18.36"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.18.36"
∷ word (ἔ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.18.36"
∷ word (ἐ ∷ κ ∷ []) "John.18.36"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.18.36"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ υ ∷ []) "John.18.36"
∷ word (τ ∷ ο ∷ ύ ∷ τ ∷ ο ∷ υ ∷ []) "John.18.36"
∷ word (ε ∷ ἰ ∷ []) "John.18.36"
∷ word (ἐ ∷ κ ∷ []) "John.18.36"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.18.36"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ υ ∷ []) "John.18.36"
∷ word (τ ∷ ο ∷ ύ ∷ τ ∷ ο ∷ υ ∷ []) "John.18.36"
∷ word (ἦ ∷ ν ∷ []) "John.18.36"
∷ word (ἡ ∷ []) "John.18.36"
∷ word (β ∷ α ∷ σ ∷ ι ∷ ∙λ ∷ ε ∷ ί ∷ α ∷ []) "John.18.36"
∷ word (ἡ ∷ []) "John.18.36"
∷ word (ἐ ∷ μ ∷ ή ∷ []) "John.18.36"
∷ word (ο ∷ ἱ ∷ []) "John.18.36"
∷ word (ὑ ∷ π ∷ η ∷ ρ ∷ έ ∷ τ ∷ α ∷ ι ∷ []) "John.18.36"
∷ word (ο ∷ ἱ ∷ []) "John.18.36"
∷ word (ἐ ∷ μ ∷ ο ∷ ὶ ∷ []) "John.18.36"
∷ word (ἠ ∷ γ ∷ ω ∷ ν ∷ ί ∷ ζ ∷ ο ∷ ν ∷ τ ∷ ο ∷ []) "John.18.36"
∷ word (ἄ ∷ ν ∷ []) "John.18.36"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.18.36"
∷ word (μ ∷ ὴ ∷ []) "John.18.36"
∷ word (π ∷ α ∷ ρ ∷ α ∷ δ ∷ ο ∷ θ ∷ ῶ ∷ []) "John.18.36"
∷ word (τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.18.36"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ί ∷ ο ∷ ι ∷ ς ∷ []) "John.18.36"
∷ word (ν ∷ ῦ ∷ ν ∷ []) "John.18.36"
∷ word (δ ∷ ὲ ∷ []) "John.18.36"
∷ word (ἡ ∷ []) "John.18.36"
∷ word (β ∷ α ∷ σ ∷ ι ∷ ∙λ ∷ ε ∷ ί ∷ α ∷ []) "John.18.36"
∷ word (ἡ ∷ []) "John.18.36"
∷ word (ἐ ∷ μ ∷ ὴ ∷ []) "John.18.36"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.18.36"
∷ word (ἔ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.18.36"
∷ word (ἐ ∷ ν ∷ τ ∷ ε ∷ ῦ ∷ θ ∷ ε ∷ ν ∷ []) "John.18.36"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.18.37"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.18.37"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.18.37"
∷ word (ὁ ∷ []) "John.18.37"
∷ word (Π ∷ ι ∷ ∙λ ∷ ᾶ ∷ τ ∷ ο ∷ ς ∷ []) "John.18.37"
∷ word (Ο ∷ ὐ ∷ κ ∷ ο ∷ ῦ ∷ ν ∷ []) "John.18.37"
∷ word (β ∷ α ∷ σ ∷ ι ∷ ∙λ ∷ ε ∷ ὺ ∷ ς ∷ []) "John.18.37"
∷ word (ε ∷ ἶ ∷ []) "John.18.37"
∷ word (σ ∷ ύ ∷ []) "John.18.37"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.18.37"
∷ word (ὁ ∷ []) "John.18.37"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.18.37"
∷ word (Σ ∷ ὺ ∷ []) "John.18.37"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ ς ∷ []) "John.18.37"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.18.37"
∷ word (β ∷ α ∷ σ ∷ ι ∷ ∙λ ∷ ε ∷ ύ ∷ ς ∷ []) "John.18.37"
∷ word (ε ∷ ἰ ∷ μ ∷ ι ∷ []) "John.18.37"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.18.37"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.18.37"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.18.37"
∷ word (γ ∷ ε ∷ γ ∷ έ ∷ ν ∷ ν ∷ η ∷ μ ∷ α ∷ ι ∷ []) "John.18.37"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.18.37"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.18.37"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.18.37"
∷ word (ἐ ∷ ∙λ ∷ ή ∷ ∙λ ∷ υ ∷ θ ∷ α ∷ []) "John.18.37"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.18.37"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.18.37"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ ν ∷ []) "John.18.37"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.18.37"
∷ word (μ ∷ α ∷ ρ ∷ τ ∷ υ ∷ ρ ∷ ή ∷ σ ∷ ω ∷ []) "John.18.37"
∷ word (τ ∷ ῇ ∷ []) "John.18.37"
∷ word (ἀ ∷ ∙λ ∷ η ∷ θ ∷ ε ∷ ί ∷ ᾳ ∷ []) "John.18.37"
∷ word (π ∷ ᾶ ∷ ς ∷ []) "John.18.37"
∷ word (ὁ ∷ []) "John.18.37"
∷ word (ὢ ∷ ν ∷ []) "John.18.37"
∷ word (ἐ ∷ κ ∷ []) "John.18.37"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.18.37"
∷ word (ἀ ∷ ∙λ ∷ η ∷ θ ∷ ε ∷ ί ∷ α ∷ ς ∷ []) "John.18.37"
∷ word (ἀ ∷ κ ∷ ο ∷ ύ ∷ ε ∷ ι ∷ []) "John.18.37"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.18.37"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.18.37"
∷ word (φ ∷ ω ∷ ν ∷ ῆ ∷ ς ∷ []) "John.18.37"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.18.38"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.18.38"
∷ word (ὁ ∷ []) "John.18.38"
∷ word (Π ∷ ι ∷ ∙λ ∷ ᾶ ∷ τ ∷ ο ∷ ς ∷ []) "John.18.38"
∷ word (Τ ∷ ί ∷ []) "John.18.38"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.18.38"
∷ word (ἀ ∷ ∙λ ∷ ή ∷ θ ∷ ε ∷ ι ∷ α ∷ []) "John.18.38"
∷ word (Κ ∷ α ∷ ὶ ∷ []) "John.18.38"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.18.38"
∷ word (ε ∷ ἰ ∷ π ∷ ὼ ∷ ν ∷ []) "John.18.38"
∷ word (π ∷ ά ∷ ∙λ ∷ ι ∷ ν ∷ []) "John.18.38"
∷ word (ἐ ∷ ξ ∷ ῆ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.18.38"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.18.38"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.18.38"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ί ∷ ο ∷ υ ∷ ς ∷ []) "John.18.38"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.18.38"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.18.38"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.18.38"
∷ word (Ἐ ∷ γ ∷ ὼ ∷ []) "John.18.38"
∷ word (ο ∷ ὐ ∷ δ ∷ ε ∷ μ ∷ ί ∷ α ∷ ν ∷ []) "John.18.38"
∷ word (ε ∷ ὑ ∷ ρ ∷ ί ∷ σ ∷ κ ∷ ω ∷ []) "John.18.38"
∷ word (ἐ ∷ ν ∷ []) "John.18.38"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.18.38"
∷ word (α ∷ ἰ ∷ τ ∷ ί ∷ α ∷ ν ∷ []) "John.18.38"
∷ word (ἔ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.18.39"
∷ word (δ ∷ ὲ ∷ []) "John.18.39"
∷ word (σ ∷ υ ∷ ν ∷ ή ∷ θ ∷ ε ∷ ι ∷ α ∷ []) "John.18.39"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.18.39"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.18.39"
∷ word (ἕ ∷ ν ∷ α ∷ []) "John.18.39"
∷ word (ἀ ∷ π ∷ ο ∷ ∙λ ∷ ύ ∷ σ ∷ ω ∷ []) "John.18.39"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.18.39"
∷ word (ἐ ∷ ν ∷ []) "John.18.39"
∷ word (τ ∷ ῷ ∷ []) "John.18.39"
∷ word (π ∷ ά ∷ σ ∷ χ ∷ α ∷ []) "John.18.39"
∷ word (β ∷ ο ∷ ύ ∷ ∙λ ∷ ε ∷ σ ∷ θ ∷ ε ∷ []) "John.18.39"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.18.39"
∷ word (ἀ ∷ π ∷ ο ∷ ∙λ ∷ ύ ∷ σ ∷ ω ∷ []) "John.18.39"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.18.39"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.18.39"
∷ word (β ∷ α ∷ σ ∷ ι ∷ ∙λ ∷ έ ∷ α ∷ []) "John.18.39"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.18.39"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ί ∷ ω ∷ ν ∷ []) "John.18.39"
∷ word (ἐ ∷ κ ∷ ρ ∷ α ∷ ύ ∷ γ ∷ α ∷ σ ∷ α ∷ ν ∷ []) "John.18.40"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.18.40"
∷ word (π ∷ ά ∷ ∙λ ∷ ι ∷ ν ∷ []) "John.18.40"
∷ word (∙λ ∷ έ ∷ γ ∷ ο ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.18.40"
∷ word (Μ ∷ ὴ ∷ []) "John.18.40"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ ν ∷ []) "John.18.40"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.18.40"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.18.40"
∷ word (Β ∷ α ∷ ρ ∷ α ∷ β ∷ β ∷ ᾶ ∷ ν ∷ []) "John.18.40"
∷ word (ἦ ∷ ν ∷ []) "John.18.40"
∷ word (δ ∷ ὲ ∷ []) "John.18.40"
∷ word (ὁ ∷ []) "John.18.40"
∷ word (Β ∷ α ∷ ρ ∷ α ∷ β ∷ β ∷ ᾶ ∷ ς ∷ []) "John.18.40"
∷ word (∙λ ∷ ῃ ∷ σ ∷ τ ∷ ή ∷ ς ∷ []) "John.18.40"
∷ word (Τ ∷ ό ∷ τ ∷ ε ∷ []) "John.19.1"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.19.1"
∷ word (ἔ ∷ ∙λ ∷ α ∷ β ∷ ε ∷ ν ∷ []) "John.19.1"
∷ word (ὁ ∷ []) "John.19.1"
∷ word (Π ∷ ι ∷ ∙λ ∷ ᾶ ∷ τ ∷ ο ∷ ς ∷ []) "John.19.1"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.19.1"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ν ∷ []) "John.19.1"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.19.1"
∷ word (ἐ ∷ μ ∷ α ∷ σ ∷ τ ∷ ί ∷ γ ∷ ω ∷ σ ∷ ε ∷ ν ∷ []) "John.19.1"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.19.2"
∷ word (ο ∷ ἱ ∷ []) "John.19.2"
∷ word (σ ∷ τ ∷ ρ ∷ α ∷ τ ∷ ι ∷ ῶ ∷ τ ∷ α ∷ ι ∷ []) "John.19.2"
∷ word (π ∷ ∙λ ∷ έ ∷ ξ ∷ α ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.19.2"
∷ word (σ ∷ τ ∷ έ ∷ φ ∷ α ∷ ν ∷ ο ∷ ν ∷ []) "John.19.2"
∷ word (ἐ ∷ ξ ∷ []) "John.19.2"
∷ word (ἀ ∷ κ ∷ α ∷ ν ∷ θ ∷ ῶ ∷ ν ∷ []) "John.19.2"
∷ word (ἐ ∷ π ∷ έ ∷ θ ∷ η ∷ κ ∷ α ∷ ν ∷ []) "John.19.2"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.19.2"
∷ word (τ ∷ ῇ ∷ []) "John.19.2"
∷ word (κ ∷ ε ∷ φ ∷ α ∷ ∙λ ∷ ῇ ∷ []) "John.19.2"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.19.2"
∷ word (ἱ ∷ μ ∷ ά ∷ τ ∷ ι ∷ ο ∷ ν ∷ []) "John.19.2"
∷ word (π ∷ ο ∷ ρ ∷ φ ∷ υ ∷ ρ ∷ ο ∷ ῦ ∷ ν ∷ []) "John.19.2"
∷ word (π ∷ ε ∷ ρ ∷ ι ∷ έ ∷ β ∷ α ∷ ∙λ ∷ ο ∷ ν ∷ []) "John.19.2"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.19.2"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.19.3"
∷ word (ἤ ∷ ρ ∷ χ ∷ ο ∷ ν ∷ τ ∷ ο ∷ []) "John.19.3"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.19.3"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.19.3"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.19.3"
∷ word (ἔ ∷ ∙λ ∷ ε ∷ γ ∷ ο ∷ ν ∷ []) "John.19.3"
∷ word (Χ ∷ α ∷ ῖ ∷ ρ ∷ ε ∷ []) "John.19.3"
∷ word (ὁ ∷ []) "John.19.3"
∷ word (β ∷ α ∷ σ ∷ ι ∷ ∙λ ∷ ε ∷ ὺ ∷ ς ∷ []) "John.19.3"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.19.3"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ί ∷ ω ∷ ν ∷ []) "John.19.3"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.19.3"
∷ word (ἐ ∷ δ ∷ ί ∷ δ ∷ ο ∷ σ ∷ α ∷ ν ∷ []) "John.19.3"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.19.3"
∷ word (ῥ ∷ α ∷ π ∷ ί ∷ σ ∷ μ ∷ α ∷ τ ∷ α ∷ []) "John.19.3"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.19.4"
∷ word (ἐ ∷ ξ ∷ ῆ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.19.4"
∷ word (π ∷ ά ∷ ∙λ ∷ ι ∷ ν ∷ []) "John.19.4"
∷ word (ἔ ∷ ξ ∷ ω ∷ []) "John.19.4"
∷ word (ὁ ∷ []) "John.19.4"
∷ word (Π ∷ ι ∷ ∙λ ∷ ᾶ ∷ τ ∷ ο ∷ ς ∷ []) "John.19.4"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.19.4"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.19.4"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.19.4"
∷ word (Ἴ ∷ δ ∷ ε ∷ []) "John.19.4"
∷ word (ἄ ∷ γ ∷ ω ∷ []) "John.19.4"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.19.4"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.19.4"
∷ word (ἔ ∷ ξ ∷ ω ∷ []) "John.19.4"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.19.4"
∷ word (γ ∷ ν ∷ ῶ ∷ τ ∷ ε ∷ []) "John.19.4"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.19.4"
∷ word (ο ∷ ὐ ∷ δ ∷ ε ∷ μ ∷ ί ∷ α ∷ ν ∷ []) "John.19.4"
∷ word (α ∷ ἰ ∷ τ ∷ ί ∷ α ∷ ν ∷ []) "John.19.4"
∷ word (ε ∷ ὑ ∷ ρ ∷ ί ∷ σ ∷ κ ∷ ω ∷ []) "John.19.4"
∷ word (ἐ ∷ ν ∷ []) "John.19.4"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.19.4"
∷ word (ἐ ∷ ξ ∷ ῆ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.19.5"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.19.5"
∷ word (ὁ ∷ []) "John.19.5"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.19.5"
∷ word (ἔ ∷ ξ ∷ ω ∷ []) "John.19.5"
∷ word (φ ∷ ο ∷ ρ ∷ ῶ ∷ ν ∷ []) "John.19.5"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.19.5"
∷ word (ἀ ∷ κ ∷ ά ∷ ν ∷ θ ∷ ι ∷ ν ∷ ο ∷ ν ∷ []) "John.19.5"
∷ word (σ ∷ τ ∷ έ ∷ φ ∷ α ∷ ν ∷ ο ∷ ν ∷ []) "John.19.5"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.19.5"
∷ word (τ ∷ ὸ ∷ []) "John.19.5"
∷ word (π ∷ ο ∷ ρ ∷ φ ∷ υ ∷ ρ ∷ ο ∷ ῦ ∷ ν ∷ []) "John.19.5"
∷ word (ἱ ∷ μ ∷ ά ∷ τ ∷ ι ∷ ο ∷ ν ∷ []) "John.19.5"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.19.5"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.19.5"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.19.5"
∷ word (Ἰ ∷ δ ∷ ο ∷ ὺ ∷ []) "John.19.5"
∷ word (ὁ ∷ []) "John.19.5"
∷ word (ἄ ∷ ν ∷ θ ∷ ρ ∷ ω ∷ π ∷ ο ∷ ς ∷ []) "John.19.5"
∷ word (ὅ ∷ τ ∷ ε ∷ []) "John.19.6"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.19.6"
∷ word (ε ∷ ἶ ∷ δ ∷ ο ∷ ν ∷ []) "John.19.6"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.19.6"
∷ word (ο ∷ ἱ ∷ []) "John.19.6"
∷ word (ἀ ∷ ρ ∷ χ ∷ ι ∷ ε ∷ ρ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.19.6"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.19.6"
∷ word (ο ∷ ἱ ∷ []) "John.19.6"
∷ word (ὑ ∷ π ∷ η ∷ ρ ∷ έ ∷ τ ∷ α ∷ ι ∷ []) "John.19.6"
∷ word (ἐ ∷ κ ∷ ρ ∷ α ∷ ύ ∷ γ ∷ α ∷ σ ∷ α ∷ ν ∷ []) "John.19.6"
∷ word (∙λ ∷ έ ∷ γ ∷ ο ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.19.6"
∷ word (Σ ∷ τ ∷ α ∷ ύ ∷ ρ ∷ ω ∷ σ ∷ ο ∷ ν ∷ []) "John.19.6"
∷ word (σ ∷ τ ∷ α ∷ ύ ∷ ρ ∷ ω ∷ σ ∷ ο ∷ ν ∷ []) "John.19.6"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.19.6"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.19.6"
∷ word (ὁ ∷ []) "John.19.6"
∷ word (Π ∷ ι ∷ ∙λ ∷ ᾶ ∷ τ ∷ ο ∷ ς ∷ []) "John.19.6"
∷ word (Λ ∷ ά ∷ β ∷ ε ∷ τ ∷ ε ∷ []) "John.19.6"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.19.6"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.19.6"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.19.6"
∷ word (σ ∷ τ ∷ α ∷ υ ∷ ρ ∷ ώ ∷ σ ∷ α ∷ τ ∷ ε ∷ []) "John.19.6"
∷ word (ἐ ∷ γ ∷ ὼ ∷ []) "John.19.6"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.19.6"
∷ word (ο ∷ ὐ ∷ χ ∷ []) "John.19.6"
∷ word (ε ∷ ὑ ∷ ρ ∷ ί ∷ σ ∷ κ ∷ ω ∷ []) "John.19.6"
∷ word (ἐ ∷ ν ∷ []) "John.19.6"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.19.6"
∷ word (α ∷ ἰ ∷ τ ∷ ί ∷ α ∷ ν ∷ []) "John.19.6"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.19.7"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.19.7"
∷ word (ο ∷ ἱ ∷ []) "John.19.7"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ῖ ∷ ο ∷ ι ∷ []) "John.19.7"
∷ word (Ἡ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.19.7"
∷ word (ν ∷ ό ∷ μ ∷ ο ∷ ν ∷ []) "John.19.7"
∷ word (ἔ ∷ χ ∷ ο ∷ μ ∷ ε ∷ ν ∷ []) "John.19.7"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.19.7"
∷ word (κ ∷ α ∷ τ ∷ ὰ ∷ []) "John.19.7"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.19.7"
∷ word (ν ∷ ό ∷ μ ∷ ο ∷ ν ∷ []) "John.19.7"
∷ word (ὀ ∷ φ ∷ ε ∷ ί ∷ ∙λ ∷ ε ∷ ι ∷ []) "John.19.7"
∷ word (ἀ ∷ π ∷ ο ∷ θ ∷ α ∷ ν ∷ ε ∷ ῖ ∷ ν ∷ []) "John.19.7"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.19.7"
∷ word (υ ∷ ἱ ∷ ὸ ∷ ν ∷ []) "John.19.7"
∷ word (θ ∷ ε ∷ ο ∷ ῦ ∷ []) "John.19.7"
∷ word (ἑ ∷ α ∷ υ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.19.7"
∷ word (ἐ ∷ π ∷ ο ∷ ί ∷ η ∷ σ ∷ ε ∷ ν ∷ []) "John.19.7"
∷ word (Ὅ ∷ τ ∷ ε ∷ []) "John.19.8"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.19.8"
∷ word (ἤ ∷ κ ∷ ο ∷ υ ∷ σ ∷ ε ∷ ν ∷ []) "John.19.8"
∷ word (ὁ ∷ []) "John.19.8"
∷ word (Π ∷ ι ∷ ∙λ ∷ ᾶ ∷ τ ∷ ο ∷ ς ∷ []) "John.19.8"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ ν ∷ []) "John.19.8"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.19.8"
∷ word (∙λ ∷ ό ∷ γ ∷ ο ∷ ν ∷ []) "John.19.8"
∷ word (μ ∷ ᾶ ∷ ∙λ ∷ ∙λ ∷ ο ∷ ν ∷ []) "John.19.8"
∷ word (ἐ ∷ φ ∷ ο ∷ β ∷ ή ∷ θ ∷ η ∷ []) "John.19.8"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.19.9"
∷ word (ε ∷ ἰ ∷ σ ∷ ῆ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.19.9"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.19.9"
∷ word (τ ∷ ὸ ∷ []) "John.19.9"
∷ word (π ∷ ρ ∷ α ∷ ι ∷ τ ∷ ώ ∷ ρ ∷ ι ∷ ο ∷ ν ∷ []) "John.19.9"
∷ word (π ∷ ά ∷ ∙λ ∷ ι ∷ ν ∷ []) "John.19.9"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.19.9"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.19.9"
∷ word (τ ∷ ῷ ∷ []) "John.19.9"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ []) "John.19.9"
∷ word (Π ∷ ό ∷ θ ∷ ε ∷ ν ∷ []) "John.19.9"
∷ word (ε ∷ ἶ ∷ []) "John.19.9"
∷ word (σ ∷ ύ ∷ []) "John.19.9"
∷ word (ὁ ∷ []) "John.19.9"
∷ word (δ ∷ ὲ ∷ []) "John.19.9"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.19.9"
∷ word (ἀ ∷ π ∷ ό ∷ κ ∷ ρ ∷ ι ∷ σ ∷ ι ∷ ν ∷ []) "John.19.9"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.19.9"
∷ word (ἔ ∷ δ ∷ ω ∷ κ ∷ ε ∷ ν ∷ []) "John.19.9"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.19.9"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.19.10"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.19.10"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.19.10"
∷ word (ὁ ∷ []) "John.19.10"
∷ word (Π ∷ ι ∷ ∙λ ∷ ᾶ ∷ τ ∷ ο ∷ ς ∷ []) "John.19.10"
∷ word (Ἐ ∷ μ ∷ ο ∷ ὶ ∷ []) "John.19.10"
∷ word (ο ∷ ὐ ∷ []) "John.19.10"
∷ word (∙λ ∷ α ∷ ∙λ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.19.10"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.19.10"
∷ word (ο ∷ ἶ ∷ δ ∷ α ∷ ς ∷ []) "John.19.10"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.19.10"
∷ word (ἐ ∷ ξ ∷ ο ∷ υ ∷ σ ∷ ί ∷ α ∷ ν ∷ []) "John.19.10"
∷ word (ἔ ∷ χ ∷ ω ∷ []) "John.19.10"
∷ word (ἀ ∷ π ∷ ο ∷ ∙λ ∷ ῦ ∷ σ ∷ α ∷ ί ∷ []) "John.19.10"
∷ word (σ ∷ ε ∷ []) "John.19.10"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.19.10"
∷ word (ἐ ∷ ξ ∷ ο ∷ υ ∷ σ ∷ ί ∷ α ∷ ν ∷ []) "John.19.10"
∷ word (ἔ ∷ χ ∷ ω ∷ []) "John.19.10"
∷ word (σ ∷ τ ∷ α ∷ υ ∷ ρ ∷ ῶ ∷ σ ∷ α ∷ ί ∷ []) "John.19.10"
∷ word (σ ∷ ε ∷ []) "John.19.10"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.19.11"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.19.11"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.19.11"
∷ word (Ο ∷ ὐ ∷ κ ∷ []) "John.19.11"
∷ word (ε ∷ ἶ ∷ χ ∷ ε ∷ ς ∷ []) "John.19.11"
∷ word (ἐ ∷ ξ ∷ ο ∷ υ ∷ σ ∷ ί ∷ α ∷ ν ∷ []) "John.19.11"
∷ word (κ ∷ α ∷ τ ∷ []) "John.19.11"
∷ word (ἐ ∷ μ ∷ ο ∷ ῦ ∷ []) "John.19.11"
∷ word (ο ∷ ὐ ∷ δ ∷ ε ∷ μ ∷ ί ∷ α ∷ ν ∷ []) "John.19.11"
∷ word (ε ∷ ἰ ∷ []) "John.19.11"
∷ word (μ ∷ ὴ ∷ []) "John.19.11"
∷ word (ἦ ∷ ν ∷ []) "John.19.11"
∷ word (δ ∷ ε ∷ δ ∷ ο ∷ μ ∷ έ ∷ ν ∷ ο ∷ ν ∷ []) "John.19.11"
∷ word (σ ∷ ο ∷ ι ∷ []) "John.19.11"
∷ word (ἄ ∷ ν ∷ ω ∷ θ ∷ ε ∷ ν ∷ []) "John.19.11"
∷ word (δ ∷ ι ∷ ὰ ∷ []) "John.19.11"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.19.11"
∷ word (ὁ ∷ []) "John.19.11"
∷ word (π ∷ α ∷ ρ ∷ α ∷ δ ∷ ο ∷ ύ ∷ ς ∷ []) "John.19.11"
∷ word (μ ∷ έ ∷ []) "John.19.11"
∷ word (σ ∷ ο ∷ ι ∷ []) "John.19.11"
∷ word (μ ∷ ε ∷ ί ∷ ζ ∷ ο ∷ ν ∷ α ∷ []) "John.19.11"
∷ word (ἁ ∷ μ ∷ α ∷ ρ ∷ τ ∷ ί ∷ α ∷ ν ∷ []) "John.19.11"
∷ word (ἔ ∷ χ ∷ ε ∷ ι ∷ []) "John.19.11"
∷ word (ἐ ∷ κ ∷ []) "John.19.12"
∷ word (τ ∷ ο ∷ ύ ∷ τ ∷ ο ∷ υ ∷ []) "John.19.12"
∷ word (ὁ ∷ []) "John.19.12"
∷ word (Π ∷ ι ∷ ∙λ ∷ ᾶ ∷ τ ∷ ο ∷ ς ∷ []) "John.19.12"
∷ word (ἐ ∷ ζ ∷ ή ∷ τ ∷ ε ∷ ι ∷ []) "John.19.12"
∷ word (ἀ ∷ π ∷ ο ∷ ∙λ ∷ ῦ ∷ σ ∷ α ∷ ι ∷ []) "John.19.12"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.19.12"
∷ word (ο ∷ ἱ ∷ []) "John.19.12"
∷ word (δ ∷ ὲ ∷ []) "John.19.12"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ῖ ∷ ο ∷ ι ∷ []) "John.19.12"
∷ word (ἐ ∷ κ ∷ ρ ∷ α ∷ ύ ∷ γ ∷ α ∷ σ ∷ α ∷ ν ∷ []) "John.19.12"
∷ word (∙λ ∷ έ ∷ γ ∷ ο ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.19.12"
∷ word (Ἐ ∷ ὰ ∷ ν ∷ []) "John.19.12"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ ν ∷ []) "John.19.12"
∷ word (ἀ ∷ π ∷ ο ∷ ∙λ ∷ ύ ∷ σ ∷ ῃ ∷ ς ∷ []) "John.19.12"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.19.12"
∷ word (ε ∷ ἶ ∷ []) "John.19.12"
∷ word (φ ∷ ί ∷ ∙λ ∷ ο ∷ ς ∷ []) "John.19.12"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.19.12"
∷ word (Κ ∷ α ∷ ί ∷ σ ∷ α ∷ ρ ∷ ο ∷ ς ∷ []) "John.19.12"
∷ word (π ∷ ᾶ ∷ ς ∷ []) "John.19.12"
∷ word (ὁ ∷ []) "John.19.12"
∷ word (β ∷ α ∷ σ ∷ ι ∷ ∙λ ∷ έ ∷ α ∷ []) "John.19.12"
∷ word (ἑ ∷ α ∷ υ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.19.12"
∷ word (π ∷ ο ∷ ι ∷ ῶ ∷ ν ∷ []) "John.19.12"
∷ word (ἀ ∷ ν ∷ τ ∷ ι ∷ ∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.19.12"
∷ word (τ ∷ ῷ ∷ []) "John.19.12"
∷ word (Κ ∷ α ∷ ί ∷ σ ∷ α ∷ ρ ∷ ι ∷ []) "John.19.12"
∷ word (Ὁ ∷ []) "John.19.13"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.19.13"
∷ word (Π ∷ ι ∷ ∙λ ∷ ᾶ ∷ τ ∷ ο ∷ ς ∷ []) "John.19.13"
∷ word (ἀ ∷ κ ∷ ο ∷ ύ ∷ σ ∷ α ∷ ς ∷ []) "John.19.13"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.19.13"
∷ word (∙λ ∷ ό ∷ γ ∷ ω ∷ ν ∷ []) "John.19.13"
∷ word (τ ∷ ο ∷ ύ ∷ τ ∷ ω ∷ ν ∷ []) "John.19.13"
∷ word (ἤ ∷ γ ∷ α ∷ γ ∷ ε ∷ ν ∷ []) "John.19.13"
∷ word (ἔ ∷ ξ ∷ ω ∷ []) "John.19.13"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.19.13"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ν ∷ []) "John.19.13"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.19.13"
∷ word (ἐ ∷ κ ∷ ά ∷ θ ∷ ι ∷ σ ∷ ε ∷ ν ∷ []) "John.19.13"
∷ word (ἐ ∷ π ∷ ὶ ∷ []) "John.19.13"
∷ word (β ∷ ή ∷ μ ∷ α ∷ τ ∷ ο ∷ ς ∷ []) "John.19.13"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.19.13"
∷ word (τ ∷ ό ∷ π ∷ ο ∷ ν ∷ []) "John.19.13"
∷ word (∙λ ∷ ε ∷ γ ∷ ό ∷ μ ∷ ε ∷ ν ∷ ο ∷ ν ∷ []) "John.19.13"
∷ word (Λ ∷ ι ∷ θ ∷ ό ∷ σ ∷ τ ∷ ρ ∷ ω ∷ τ ∷ ο ∷ ν ∷ []) "John.19.13"
∷ word (Ἑ ∷ β ∷ ρ ∷ α ∷ ϊ ∷ σ ∷ τ ∷ ὶ ∷ []) "John.19.13"
∷ word (δ ∷ ὲ ∷ []) "John.19.13"
∷ word (Γ ∷ α ∷ β ∷ β ∷ α ∷ θ ∷ α ∷ []) "John.19.13"
∷ word (ἦ ∷ ν ∷ []) "John.19.14"
∷ word (δ ∷ ὲ ∷ []) "John.19.14"
∷ word (π ∷ α ∷ ρ ∷ α ∷ σ ∷ κ ∷ ε ∷ υ ∷ ὴ ∷ []) "John.19.14"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.19.14"
∷ word (π ∷ ά ∷ σ ∷ χ ∷ α ∷ []) "John.19.14"
∷ word (ὥ ∷ ρ ∷ α ∷ []) "John.19.14"
∷ word (ἦ ∷ ν ∷ []) "John.19.14"
∷ word (ὡ ∷ ς ∷ []) "John.19.14"
∷ word (ἕ ∷ κ ∷ τ ∷ η ∷ []) "John.19.14"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.19.14"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.19.14"
∷ word (τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.19.14"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ί ∷ ο ∷ ι ∷ ς ∷ []) "John.19.14"
∷ word (Ἴ ∷ δ ∷ ε ∷ []) "John.19.14"
∷ word (ὁ ∷ []) "John.19.14"
∷ word (β ∷ α ∷ σ ∷ ι ∷ ∙λ ∷ ε ∷ ὺ ∷ ς ∷ []) "John.19.14"
∷ word (ὑ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.19.14"
∷ word (ἐ ∷ κ ∷ ρ ∷ α ∷ ύ ∷ γ ∷ α ∷ σ ∷ α ∷ ν ∷ []) "John.19.15"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.19.15"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ο ∷ ι ∷ []) "John.19.15"
∷ word (Ἆ ∷ ρ ∷ ο ∷ ν ∷ []) "John.19.15"
∷ word (ἆ ∷ ρ ∷ ο ∷ ν ∷ []) "John.19.15"
∷ word (σ ∷ τ ∷ α ∷ ύ ∷ ρ ∷ ω ∷ σ ∷ ο ∷ ν ∷ []) "John.19.15"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.19.15"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.19.15"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.19.15"
∷ word (ὁ ∷ []) "John.19.15"
∷ word (Π ∷ ι ∷ ∙λ ∷ ᾶ ∷ τ ∷ ο ∷ ς ∷ []) "John.19.15"
∷ word (Τ ∷ ὸ ∷ ν ∷ []) "John.19.15"
∷ word (β ∷ α ∷ σ ∷ ι ∷ ∙λ ∷ έ ∷ α ∷ []) "John.19.15"
∷ word (ὑ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.19.15"
∷ word (σ ∷ τ ∷ α ∷ υ ∷ ρ ∷ ώ ∷ σ ∷ ω ∷ []) "John.19.15"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.19.15"
∷ word (ο ∷ ἱ ∷ []) "John.19.15"
∷ word (ἀ ∷ ρ ∷ χ ∷ ι ∷ ε ∷ ρ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.19.15"
∷ word (Ο ∷ ὐ ∷ κ ∷ []) "John.19.15"
∷ word (ἔ ∷ χ ∷ ο ∷ μ ∷ ε ∷ ν ∷ []) "John.19.15"
∷ word (β ∷ α ∷ σ ∷ ι ∷ ∙λ ∷ έ ∷ α ∷ []) "John.19.15"
∷ word (ε ∷ ἰ ∷ []) "John.19.15"
∷ word (μ ∷ ὴ ∷ []) "John.19.15"
∷ word (Κ ∷ α ∷ ί ∷ σ ∷ α ∷ ρ ∷ α ∷ []) "John.19.15"
∷ word (τ ∷ ό ∷ τ ∷ ε ∷ []) "John.19.16"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.19.16"
∷ word (π ∷ α ∷ ρ ∷ έ ∷ δ ∷ ω ∷ κ ∷ ε ∷ ν ∷ []) "John.19.16"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.19.16"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.19.16"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.19.16"
∷ word (σ ∷ τ ∷ α ∷ υ ∷ ρ ∷ ω ∷ θ ∷ ῇ ∷ []) "John.19.16"
∷ word (Π ∷ α ∷ ρ ∷ έ ∷ ∙λ ∷ α ∷ β ∷ ο ∷ ν ∷ []) "John.19.16"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.19.16"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.19.16"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ν ∷ []) "John.19.16"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.19.17"
∷ word (β ∷ α ∷ σ ∷ τ ∷ ά ∷ ζ ∷ ω ∷ ν ∷ []) "John.19.17"
∷ word (α ∷ ὑ ∷ τ ∷ ῷ ∷ []) "John.19.17"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.19.17"
∷ word (σ ∷ τ ∷ α ∷ υ ∷ ρ ∷ ὸ ∷ ν ∷ []) "John.19.17"
∷ word (ἐ ∷ ξ ∷ ῆ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.19.17"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.19.17"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.19.17"
∷ word (∙λ ∷ ε ∷ γ ∷ ό ∷ μ ∷ ε ∷ ν ∷ ο ∷ ν ∷ []) "John.19.17"
∷ word (Κ ∷ ρ ∷ α ∷ ν ∷ ί ∷ ο ∷ υ ∷ []) "John.19.17"
∷ word (Τ ∷ ό ∷ π ∷ ο ∷ ν ∷ []) "John.19.17"
∷ word (ὃ ∷ []) "John.19.17"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.19.17"
∷ word (Ἑ ∷ β ∷ ρ ∷ α ∷ ϊ ∷ σ ∷ τ ∷ ὶ ∷ []) "John.19.17"
∷ word (Γ ∷ ο ∷ ∙λ ∷ γ ∷ ο ∷ θ ∷ α ∷ []) "John.19.17"
∷ word (ὅ ∷ π ∷ ο ∷ υ ∷ []) "John.19.18"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.19.18"
∷ word (ἐ ∷ σ ∷ τ ∷ α ∷ ύ ∷ ρ ∷ ω ∷ σ ∷ α ∷ ν ∷ []) "John.19.18"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.19.18"
∷ word (μ ∷ ε ∷ τ ∷ []) "John.19.18"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.19.18"
∷ word (ἄ ∷ ∙λ ∷ ∙λ ∷ ο ∷ υ ∷ ς ∷ []) "John.19.18"
∷ word (δ ∷ ύ ∷ ο ∷ []) "John.19.18"
∷ word (ἐ ∷ ν ∷ τ ∷ ε ∷ ῦ ∷ θ ∷ ε ∷ ν ∷ []) "John.19.18"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.19.18"
∷ word (ἐ ∷ ν ∷ τ ∷ ε ∷ ῦ ∷ θ ∷ ε ∷ ν ∷ []) "John.19.18"
∷ word (μ ∷ έ ∷ σ ∷ ο ∷ ν ∷ []) "John.19.18"
∷ word (δ ∷ ὲ ∷ []) "John.19.18"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.19.18"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ν ∷ []) "John.19.18"
∷ word (ἔ ∷ γ ∷ ρ ∷ α ∷ ψ ∷ ε ∷ ν ∷ []) "John.19.19"
∷ word (δ ∷ ὲ ∷ []) "John.19.19"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.19.19"
∷ word (τ ∷ ί ∷ τ ∷ ∙λ ∷ ο ∷ ν ∷ []) "John.19.19"
∷ word (ὁ ∷ []) "John.19.19"
∷ word (Π ∷ ι ∷ ∙λ ∷ ᾶ ∷ τ ∷ ο ∷ ς ∷ []) "John.19.19"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.19.19"
∷ word (ἔ ∷ θ ∷ η ∷ κ ∷ ε ∷ ν ∷ []) "John.19.19"
∷ word (ἐ ∷ π ∷ ὶ ∷ []) "John.19.19"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.19.19"
∷ word (σ ∷ τ ∷ α ∷ υ ∷ ρ ∷ ο ∷ ῦ ∷ []) "John.19.19"
∷ word (ἦ ∷ ν ∷ []) "John.19.19"
∷ word (δ ∷ ὲ ∷ []) "John.19.19"
∷ word (γ ∷ ε ∷ γ ∷ ρ ∷ α ∷ μ ∷ μ ∷ έ ∷ ν ∷ ο ∷ ν ∷ []) "John.19.19"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.19.19"
∷ word (ὁ ∷ []) "John.19.19"
∷ word (Ν ∷ α ∷ ζ ∷ ω ∷ ρ ∷ α ∷ ῖ ∷ ο ∷ ς ∷ []) "John.19.19"
∷ word (ὁ ∷ []) "John.19.19"
∷ word (β ∷ α ∷ σ ∷ ι ∷ ∙λ ∷ ε ∷ ὺ ∷ ς ∷ []) "John.19.19"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.19.19"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ί ∷ ω ∷ ν ∷ []) "John.19.19"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ ν ∷ []) "John.19.20"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.19.20"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.19.20"
∷ word (τ ∷ ί ∷ τ ∷ ∙λ ∷ ο ∷ ν ∷ []) "John.19.20"
∷ word (π ∷ ο ∷ ∙λ ∷ ∙λ ∷ ο ∷ ὶ ∷ []) "John.19.20"
∷ word (ἀ ∷ ν ∷ έ ∷ γ ∷ ν ∷ ω ∷ σ ∷ α ∷ ν ∷ []) "John.19.20"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.19.20"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ί ∷ ω ∷ ν ∷ []) "John.19.20"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.19.20"
∷ word (ἐ ∷ γ ∷ γ ∷ ὺ ∷ ς ∷ []) "John.19.20"
∷ word (ἦ ∷ ν ∷ []) "John.19.20"
∷ word (ὁ ∷ []) "John.19.20"
∷ word (τ ∷ ό ∷ π ∷ ο ∷ ς ∷ []) "John.19.20"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.19.20"
∷ word (π ∷ ό ∷ ∙λ ∷ ε ∷ ω ∷ ς ∷ []) "John.19.20"
∷ word (ὅ ∷ π ∷ ο ∷ υ ∷ []) "John.19.20"
∷ word (ἐ ∷ σ ∷ τ ∷ α ∷ υ ∷ ρ ∷ ώ ∷ θ ∷ η ∷ []) "John.19.20"
∷ word (ὁ ∷ []) "John.19.20"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.19.20"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.19.20"
∷ word (ἦ ∷ ν ∷ []) "John.19.20"
∷ word (γ ∷ ε ∷ γ ∷ ρ ∷ α ∷ μ ∷ μ ∷ έ ∷ ν ∷ ο ∷ ν ∷ []) "John.19.20"
∷ word (Ἑ ∷ β ∷ ρ ∷ α ∷ ϊ ∷ σ ∷ τ ∷ ί ∷ []) "John.19.20"
∷ word (Ῥ ∷ ω ∷ μ ∷ α ∷ ϊ ∷ σ ∷ τ ∷ ί ∷ []) "John.19.20"
∷ word (Ἑ ∷ ∙λ ∷ ∙λ ∷ η ∷ ν ∷ ι ∷ σ ∷ τ ∷ ί ∷ []) "John.19.20"
∷ word (ἔ ∷ ∙λ ∷ ε ∷ γ ∷ ο ∷ ν ∷ []) "John.19.21"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.19.21"
∷ word (τ ∷ ῷ ∷ []) "John.19.21"
∷ word (Π ∷ ι ∷ ∙λ ∷ ά ∷ τ ∷ ῳ ∷ []) "John.19.21"
∷ word (ο ∷ ἱ ∷ []) "John.19.21"
∷ word (ἀ ∷ ρ ∷ χ ∷ ι ∷ ε ∷ ρ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.19.21"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.19.21"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ί ∷ ω ∷ ν ∷ []) "John.19.21"
∷ word (Μ ∷ ὴ ∷ []) "John.19.21"
∷ word (γ ∷ ρ ∷ ά ∷ φ ∷ ε ∷ []) "John.19.21"
∷ word (Ὁ ∷ []) "John.19.21"
∷ word (β ∷ α ∷ σ ∷ ι ∷ ∙λ ∷ ε ∷ ὺ ∷ ς ∷ []) "John.19.21"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.19.21"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ί ∷ ω ∷ ν ∷ []) "John.19.21"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ []) "John.19.21"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.19.21"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ο ∷ ς ∷ []) "John.19.21"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.19.21"
∷ word (Β ∷ α ∷ σ ∷ ι ∷ ∙λ ∷ ε ∷ ὺ ∷ ς ∷ []) "John.19.21"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.19.21"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ί ∷ ω ∷ ν ∷ []) "John.19.21"
∷ word (ε ∷ ἰ ∷ μ ∷ ί ∷ []) "John.19.21"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.19.22"
∷ word (ὁ ∷ []) "John.19.22"
∷ word (Π ∷ ι ∷ ∙λ ∷ ᾶ ∷ τ ∷ ο ∷ ς ∷ []) "John.19.22"
∷ word (Ὃ ∷ []) "John.19.22"
∷ word (γ ∷ έ ∷ γ ∷ ρ ∷ α ∷ φ ∷ α ∷ []) "John.19.22"
∷ word (γ ∷ έ ∷ γ ∷ ρ ∷ α ∷ φ ∷ α ∷ []) "John.19.22"
∷ word (ο ∷ ἱ ∷ []) "John.19.23"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.19.23"
∷ word (σ ∷ τ ∷ ρ ∷ α ∷ τ ∷ ι ∷ ῶ ∷ τ ∷ α ∷ ι ∷ []) "John.19.23"
∷ word (ὅ ∷ τ ∷ ε ∷ []) "John.19.23"
∷ word (ἐ ∷ σ ∷ τ ∷ α ∷ ύ ∷ ρ ∷ ω ∷ σ ∷ α ∷ ν ∷ []) "John.19.23"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.19.23"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ν ∷ []) "John.19.23"
∷ word (ἔ ∷ ∙λ ∷ α ∷ β ∷ ο ∷ ν ∷ []) "John.19.23"
∷ word (τ ∷ ὰ ∷ []) "John.19.23"
∷ word (ἱ ∷ μ ∷ ά ∷ τ ∷ ι ∷ α ∷ []) "John.19.23"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.19.23"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.19.23"
∷ word (ἐ ∷ π ∷ ο ∷ ί ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.19.23"
∷ word (τ ∷ έ ∷ σ ∷ σ ∷ α ∷ ρ ∷ α ∷ []) "John.19.23"
∷ word (μ ∷ έ ∷ ρ ∷ η ∷ []) "John.19.23"
∷ word (ἑ ∷ κ ∷ ά ∷ σ ∷ τ ∷ ῳ ∷ []) "John.19.23"
∷ word (σ ∷ τ ∷ ρ ∷ α ∷ τ ∷ ι ∷ ώ ∷ τ ∷ ῃ ∷ []) "John.19.23"
∷ word (μ ∷ έ ∷ ρ ∷ ο ∷ ς ∷ []) "John.19.23"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.19.23"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.19.23"
∷ word (χ ∷ ι ∷ τ ∷ ῶ ∷ ν ∷ α ∷ []) "John.19.23"
∷ word (ἦ ∷ ν ∷ []) "John.19.23"
∷ word (δ ∷ ὲ ∷ []) "John.19.23"
∷ word (ὁ ∷ []) "John.19.23"
∷ word (χ ∷ ι ∷ τ ∷ ὼ ∷ ν ∷ []) "John.19.23"
∷ word (ἄ ∷ ρ ∷ α ∷ φ ∷ ο ∷ ς ∷ []) "John.19.23"
∷ word (ἐ ∷ κ ∷ []) "John.19.23"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.19.23"
∷ word (ἄ ∷ ν ∷ ω ∷ θ ∷ ε ∷ ν ∷ []) "John.19.23"
∷ word (ὑ ∷ φ ∷ α ∷ ν ∷ τ ∷ ὸ ∷ ς ∷ []) "John.19.23"
∷ word (δ ∷ ι ∷ []) "John.19.23"
∷ word (ὅ ∷ ∙λ ∷ ο ∷ υ ∷ []) "John.19.23"
∷ word (ε ∷ ἶ ∷ π ∷ α ∷ ν ∷ []) "John.19.24"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.19.24"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.19.24"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ή ∷ ∙λ ∷ ο ∷ υ ∷ ς ∷ []) "John.19.24"
∷ word (Μ ∷ ὴ ∷ []) "John.19.24"
∷ word (σ ∷ χ ∷ ί ∷ σ ∷ ω ∷ μ ∷ ε ∷ ν ∷ []) "John.19.24"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.19.24"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.19.24"
∷ word (∙λ ∷ ά ∷ χ ∷ ω ∷ μ ∷ ε ∷ ν ∷ []) "John.19.24"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.19.24"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.19.24"
∷ word (τ ∷ ί ∷ ν ∷ ο ∷ ς ∷ []) "John.19.24"
∷ word (ἔ ∷ σ ∷ τ ∷ α ∷ ι ∷ []) "John.19.24"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.19.24"
∷ word (ἡ ∷ []) "John.19.24"
∷ word (γ ∷ ρ ∷ α ∷ φ ∷ ὴ ∷ []) "John.19.24"
∷ word (π ∷ ∙λ ∷ η ∷ ρ ∷ ω ∷ θ ∷ ῇ ∷ []) "John.19.24"
∷ word (ἡ ∷ []) "John.19.24"
∷ word (∙λ ∷ έ ∷ γ ∷ ο ∷ υ ∷ σ ∷ α ∷ []) "John.19.24"
∷ word (Δ ∷ ι ∷ ε ∷ μ ∷ ε ∷ ρ ∷ ί ∷ σ ∷ α ∷ ν ∷ τ ∷ ο ∷ []) "John.19.24"
∷ word (τ ∷ ὰ ∷ []) "John.19.24"
∷ word (ἱ ∷ μ ∷ ά ∷ τ ∷ ι ∷ ά ∷ []) "John.19.24"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.19.24"
∷ word (ἑ ∷ α ∷ υ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.19.24"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.19.24"
∷ word (ἐ ∷ π ∷ ὶ ∷ []) "John.19.24"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.19.24"
∷ word (ἱ ∷ μ ∷ α ∷ τ ∷ ι ∷ σ ∷ μ ∷ ό ∷ ν ∷ []) "John.19.24"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.19.24"
∷ word (ἔ ∷ β ∷ α ∷ ∙λ ∷ ο ∷ ν ∷ []) "John.19.24"
∷ word (κ ∷ ∙λ ∷ ῆ ∷ ρ ∷ ο ∷ ν ∷ []) "John.19.24"
∷ word (Ο ∷ ἱ ∷ []) "John.19.24"
∷ word (μ ∷ ὲ ∷ ν ∷ []) "John.19.24"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.19.24"
∷ word (σ ∷ τ ∷ ρ ∷ α ∷ τ ∷ ι ∷ ῶ ∷ τ ∷ α ∷ ι ∷ []) "John.19.24"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.19.24"
∷ word (ἐ ∷ π ∷ ο ∷ ί ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.19.24"
∷ word (Ε ∷ ἱ ∷ σ ∷ τ ∷ ή ∷ κ ∷ ε ∷ ι ∷ σ ∷ α ∷ ν ∷ []) "John.19.25"
∷ word (δ ∷ ὲ ∷ []) "John.19.25"
∷ word (π ∷ α ∷ ρ ∷ ὰ ∷ []) "John.19.25"
∷ word (τ ∷ ῷ ∷ []) "John.19.25"
∷ word (σ ∷ τ ∷ α ∷ υ ∷ ρ ∷ ῷ ∷ []) "John.19.25"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.19.25"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ []) "John.19.25"
∷ word (ἡ ∷ []) "John.19.25"
∷ word (μ ∷ ή ∷ τ ∷ η ∷ ρ ∷ []) "John.19.25"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.19.25"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.19.25"
∷ word (ἡ ∷ []) "John.19.25"
∷ word (ἀ ∷ δ ∷ ε ∷ ∙λ ∷ φ ∷ ὴ ∷ []) "John.19.25"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.19.25"
∷ word (μ ∷ η ∷ τ ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.19.25"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.19.25"
∷ word (Μ ∷ α ∷ ρ ∷ ί ∷ α ∷ []) "John.19.25"
∷ word (ἡ ∷ []) "John.19.25"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.19.25"
∷ word (Κ ∷ ∙λ ∷ ω ∷ π ∷ ᾶ ∷ []) "John.19.25"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.19.25"
∷ word (Μ ∷ α ∷ ρ ∷ ί ∷ α ∷ []) "John.19.25"
∷ word (ἡ ∷ []) "John.19.25"
∷ word (Μ ∷ α ∷ γ ∷ δ ∷ α ∷ ∙λ ∷ η ∷ ν ∷ ή ∷ []) "John.19.25"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.19.26"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.19.26"
∷ word (ἰ ∷ δ ∷ ὼ ∷ ν ∷ []) "John.19.26"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.19.26"
∷ word (μ ∷ η ∷ τ ∷ έ ∷ ρ ∷ α ∷ []) "John.19.26"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.19.26"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.19.26"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ ὴ ∷ ν ∷ []) "John.19.26"
∷ word (π ∷ α ∷ ρ ∷ ε ∷ σ ∷ τ ∷ ῶ ∷ τ ∷ α ∷ []) "John.19.26"
∷ word (ὃ ∷ ν ∷ []) "John.19.26"
∷ word (ἠ ∷ γ ∷ ά ∷ π ∷ α ∷ []) "John.19.26"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.19.26"
∷ word (τ ∷ ῇ ∷ []) "John.19.26"
∷ word (μ ∷ η ∷ τ ∷ ρ ∷ ί ∷ []) "John.19.26"
∷ word (Γ ∷ ύ ∷ ν ∷ α ∷ ι ∷ []) "John.19.26"
∷ word (ἴ ∷ δ ∷ ε ∷ []) "John.19.26"
∷ word (ὁ ∷ []) "John.19.26"
∷ word (υ ∷ ἱ ∷ ό ∷ ς ∷ []) "John.19.26"
∷ word (σ ∷ ο ∷ υ ∷ []) "John.19.26"
∷ word (ε ∷ ἶ ∷ τ ∷ α ∷ []) "John.19.27"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.19.27"
∷ word (τ ∷ ῷ ∷ []) "John.19.27"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ ῇ ∷ []) "John.19.27"
∷ word (Ἴ ∷ δ ∷ ε ∷ []) "John.19.27"
∷ word (ἡ ∷ []) "John.19.27"
∷ word (μ ∷ ή ∷ τ ∷ η ∷ ρ ∷ []) "John.19.27"
∷ word (σ ∷ ο ∷ υ ∷ []) "John.19.27"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.19.27"
∷ word (ἀ ∷ π ∷ []) "John.19.27"
∷ word (ἐ ∷ κ ∷ ε ∷ ί ∷ ν ∷ η ∷ ς ∷ []) "John.19.27"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.19.27"
∷ word (ὥ ∷ ρ ∷ α ∷ ς ∷ []) "John.19.27"
∷ word (ἔ ∷ ∙λ ∷ α ∷ β ∷ ε ∷ ν ∷ []) "John.19.27"
∷ word (ὁ ∷ []) "John.19.27"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ ὴ ∷ ς ∷ []) "John.19.27"
∷ word (α ∷ ὐ ∷ τ ∷ ὴ ∷ ν ∷ []) "John.19.27"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.19.27"
∷ word (τ ∷ ὰ ∷ []) "John.19.27"
∷ word (ἴ ∷ δ ∷ ι ∷ α ∷ []) "John.19.27"
∷ word (Μ ∷ ε ∷ τ ∷ ὰ ∷ []) "John.19.28"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.19.28"
∷ word (ε ∷ ἰ ∷ δ ∷ ὼ ∷ ς ∷ []) "John.19.28"
∷ word (ὁ ∷ []) "John.19.28"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.19.28"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.19.28"
∷ word (ἤ ∷ δ ∷ η ∷ []) "John.19.28"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ α ∷ []) "John.19.28"
∷ word (τ ∷ ε ∷ τ ∷ έ ∷ ∙λ ∷ ε ∷ σ ∷ τ ∷ α ∷ ι ∷ []) "John.19.28"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.19.28"
∷ word (τ ∷ ε ∷ ∙λ ∷ ε ∷ ι ∷ ω ∷ θ ∷ ῇ ∷ []) "John.19.28"
∷ word (ἡ ∷ []) "John.19.28"
∷ word (γ ∷ ρ ∷ α ∷ φ ∷ ὴ ∷ []) "John.19.28"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.19.28"
∷ word (Δ ∷ ι ∷ ψ ∷ ῶ ∷ []) "John.19.28"
∷ word (σ ∷ κ ∷ ε ∷ ῦ ∷ ο ∷ ς ∷ []) "John.19.29"
∷ word (ἔ ∷ κ ∷ ε ∷ ι ∷ τ ∷ ο ∷ []) "John.19.29"
∷ word (ὄ ∷ ξ ∷ ο ∷ υ ∷ ς ∷ []) "John.19.29"
∷ word (μ ∷ ε ∷ σ ∷ τ ∷ ό ∷ ν ∷ []) "John.19.29"
∷ word (σ ∷ π ∷ ό ∷ γ ∷ γ ∷ ο ∷ ν ∷ []) "John.19.29"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.19.29"
∷ word (μ ∷ ε ∷ σ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.19.29"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.19.29"
∷ word (ὄ ∷ ξ ∷ ο ∷ υ ∷ ς ∷ []) "John.19.29"
∷ word (ὑ ∷ σ ∷ σ ∷ ώ ∷ π ∷ ῳ ∷ []) "John.19.29"
∷ word (π ∷ ε ∷ ρ ∷ ι ∷ θ ∷ έ ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.19.29"
∷ word (π ∷ ρ ∷ ο ∷ σ ∷ ή ∷ ν ∷ ε ∷ γ ∷ κ ∷ α ∷ ν ∷ []) "John.19.29"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.19.29"
∷ word (τ ∷ ῷ ∷ []) "John.19.29"
∷ word (σ ∷ τ ∷ ό ∷ μ ∷ α ∷ τ ∷ ι ∷ []) "John.19.29"
∷ word (ὅ ∷ τ ∷ ε ∷ []) "John.19.30"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.19.30"
∷ word (ἔ ∷ ∙λ ∷ α ∷ β ∷ ε ∷ ν ∷ []) "John.19.30"
∷ word (τ ∷ ὸ ∷ []) "John.19.30"
∷ word (ὄ ∷ ξ ∷ ο ∷ ς ∷ []) "John.19.30"
∷ word (ὁ ∷ []) "John.19.30"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.19.30"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.19.30"
∷ word (Τ ∷ ε ∷ τ ∷ έ ∷ ∙λ ∷ ε ∷ σ ∷ τ ∷ α ∷ ι ∷ []) "John.19.30"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.19.30"
∷ word (κ ∷ ∙λ ∷ ί ∷ ν ∷ α ∷ ς ∷ []) "John.19.30"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.19.30"
∷ word (κ ∷ ε ∷ φ ∷ α ∷ ∙λ ∷ ὴ ∷ ν ∷ []) "John.19.30"
∷ word (π ∷ α ∷ ρ ∷ έ ∷ δ ∷ ω ∷ κ ∷ ε ∷ ν ∷ []) "John.19.30"
∷ word (τ ∷ ὸ ∷ []) "John.19.30"
∷ word (π ∷ ν ∷ ε ∷ ῦ ∷ μ ∷ α ∷ []) "John.19.30"
∷ word (Ο ∷ ἱ ∷ []) "John.19.31"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.19.31"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ῖ ∷ ο ∷ ι ∷ []) "John.19.31"
∷ word (ἐ ∷ π ∷ ε ∷ ὶ ∷ []) "John.19.31"
∷ word (π ∷ α ∷ ρ ∷ α ∷ σ ∷ κ ∷ ε ∷ υ ∷ ὴ ∷ []) "John.19.31"
∷ word (ἦ ∷ ν ∷ []) "John.19.31"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.19.31"
∷ word (μ ∷ ὴ ∷ []) "John.19.31"
∷ word (μ ∷ ε ∷ ί ∷ ν ∷ ῃ ∷ []) "John.19.31"
∷ word (ἐ ∷ π ∷ ὶ ∷ []) "John.19.31"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.19.31"
∷ word (σ ∷ τ ∷ α ∷ υ ∷ ρ ∷ ο ∷ ῦ ∷ []) "John.19.31"
∷ word (τ ∷ ὰ ∷ []) "John.19.31"
∷ word (σ ∷ ώ ∷ μ ∷ α ∷ τ ∷ α ∷ []) "John.19.31"
∷ word (ἐ ∷ ν ∷ []) "John.19.31"
∷ word (τ ∷ ῷ ∷ []) "John.19.31"
∷ word (σ ∷ α ∷ β ∷ β ∷ ά ∷ τ ∷ ῳ ∷ []) "John.19.31"
∷ word (ἦ ∷ ν ∷ []) "John.19.31"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.19.31"
∷ word (μ ∷ ε ∷ γ ∷ ά ∷ ∙λ ∷ η ∷ []) "John.19.31"
∷ word (ἡ ∷ []) "John.19.31"
∷ word (ἡ ∷ μ ∷ έ ∷ ρ ∷ α ∷ []) "John.19.31"
∷ word (ἐ ∷ κ ∷ ε ∷ ί ∷ ν ∷ ο ∷ υ ∷ []) "John.19.31"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.19.31"
∷ word (σ ∷ α ∷ β ∷ β ∷ ά ∷ τ ∷ ο ∷ υ ∷ []) "John.19.31"
∷ word (ἠ ∷ ρ ∷ ώ ∷ τ ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.19.31"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.19.31"
∷ word (Π ∷ ι ∷ ∙λ ∷ ᾶ ∷ τ ∷ ο ∷ ν ∷ []) "John.19.31"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.19.31"
∷ word (κ ∷ α ∷ τ ∷ ε ∷ α ∷ γ ∷ ῶ ∷ σ ∷ ι ∷ ν ∷ []) "John.19.31"
∷ word (α ∷ ὐ ∷ τ ∷ ῶ ∷ ν ∷ []) "John.19.31"
∷ word (τ ∷ ὰ ∷ []) "John.19.31"
∷ word (σ ∷ κ ∷ έ ∷ ∙λ ∷ η ∷ []) "John.19.31"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.19.31"
∷ word (ἀ ∷ ρ ∷ θ ∷ ῶ ∷ σ ∷ ι ∷ ν ∷ []) "John.19.31"
∷ word (ἦ ∷ ∙λ ∷ θ ∷ ο ∷ ν ∷ []) "John.19.32"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.19.32"
∷ word (ο ∷ ἱ ∷ []) "John.19.32"
∷ word (σ ∷ τ ∷ ρ ∷ α ∷ τ ∷ ι ∷ ῶ ∷ τ ∷ α ∷ ι ∷ []) "John.19.32"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.19.32"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.19.32"
∷ word (μ ∷ ὲ ∷ ν ∷ []) "John.19.32"
∷ word (π ∷ ρ ∷ ώ ∷ τ ∷ ο ∷ υ ∷ []) "John.19.32"
∷ word (κ ∷ α ∷ τ ∷ έ ∷ α ∷ ξ ∷ α ∷ ν ∷ []) "John.19.32"
∷ word (τ ∷ ὰ ∷ []) "John.19.32"
∷ word (σ ∷ κ ∷ έ ∷ ∙λ ∷ η ∷ []) "John.19.32"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.19.32"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.19.32"
∷ word (ἄ ∷ ∙λ ∷ ∙λ ∷ ο ∷ υ ∷ []) "John.19.32"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.19.32"
∷ word (σ ∷ υ ∷ σ ∷ τ ∷ α ∷ υ ∷ ρ ∷ ω ∷ θ ∷ έ ∷ ν ∷ τ ∷ ο ∷ ς ∷ []) "John.19.32"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.19.32"
∷ word (ἐ ∷ π ∷ ὶ ∷ []) "John.19.33"
∷ word (δ ∷ ὲ ∷ []) "John.19.33"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.19.33"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ν ∷ []) "John.19.33"
∷ word (ἐ ∷ ∙λ ∷ θ ∷ ό ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.19.33"
∷ word (ὡ ∷ ς ∷ []) "John.19.33"
∷ word (ε ∷ ἶ ∷ δ ∷ ο ∷ ν ∷ []) "John.19.33"
∷ word (ἤ ∷ δ ∷ η ∷ []) "John.19.33"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.19.33"
∷ word (τ ∷ ε ∷ θ ∷ ν ∷ η ∷ κ ∷ ό ∷ τ ∷ α ∷ []) "John.19.33"
∷ word (ο ∷ ὐ ∷ []) "John.19.33"
∷ word (κ ∷ α ∷ τ ∷ έ ∷ α ∷ ξ ∷ α ∷ ν ∷ []) "John.19.33"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.19.33"
∷ word (τ ∷ ὰ ∷ []) "John.19.33"
∷ word (σ ∷ κ ∷ έ ∷ ∙λ ∷ η ∷ []) "John.19.33"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ []) "John.19.34"
∷ word (ε ∷ ἷ ∷ ς ∷ []) "John.19.34"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.19.34"
∷ word (σ ∷ τ ∷ ρ ∷ α ∷ τ ∷ ι ∷ ω ∷ τ ∷ ῶ ∷ ν ∷ []) "John.19.34"
∷ word (∙λ ∷ ό ∷ γ ∷ χ ∷ ῃ ∷ []) "John.19.34"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.19.34"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.19.34"
∷ word (π ∷ ∙λ ∷ ε ∷ υ ∷ ρ ∷ ὰ ∷ ν ∷ []) "John.19.34"
∷ word (ἔ ∷ ν ∷ υ ∷ ξ ∷ ε ∷ ν ∷ []) "John.19.34"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.19.34"
∷ word (ἐ ∷ ξ ∷ ῆ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.19.34"
∷ word (ε ∷ ὐ ∷ θ ∷ ὺ ∷ ς ∷ []) "John.19.34"
∷ word (α ∷ ἷ ∷ μ ∷ α ∷ []) "John.19.34"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.19.34"
∷ word (ὕ ∷ δ ∷ ω ∷ ρ ∷ []) "John.19.34"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.19.35"
∷ word (ὁ ∷ []) "John.19.35"
∷ word (ἑ ∷ ω ∷ ρ ∷ α ∷ κ ∷ ὼ ∷ ς ∷ []) "John.19.35"
∷ word (μ ∷ ε ∷ μ ∷ α ∷ ρ ∷ τ ∷ ύ ∷ ρ ∷ η ∷ κ ∷ ε ∷ ν ∷ []) "John.19.35"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.19.35"
∷ word (ἀ ∷ ∙λ ∷ η ∷ θ ∷ ι ∷ ν ∷ ὴ ∷ []) "John.19.35"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.19.35"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.19.35"
∷ word (ἡ ∷ []) "John.19.35"
∷ word (μ ∷ α ∷ ρ ∷ τ ∷ υ ∷ ρ ∷ ί ∷ α ∷ []) "John.19.35"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.19.35"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ο ∷ ς ∷ []) "John.19.35"
∷ word (ο ∷ ἶ ∷ δ ∷ ε ∷ ν ∷ []) "John.19.35"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.19.35"
∷ word (ἀ ∷ ∙λ ∷ η ∷ θ ∷ ῆ ∷ []) "John.19.35"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.19.35"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.19.35"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.19.35"
∷ word (ὑ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.19.35"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ η ∷ τ ∷ ε ∷ []) "John.19.35"
∷ word (ἐ ∷ γ ∷ έ ∷ ν ∷ ε ∷ τ ∷ ο ∷ []) "John.19.36"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.19.36"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.19.36"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.19.36"
∷ word (ἡ ∷ []) "John.19.36"
∷ word (γ ∷ ρ ∷ α ∷ φ ∷ ὴ ∷ []) "John.19.36"
∷ word (π ∷ ∙λ ∷ η ∷ ρ ∷ ω ∷ θ ∷ ῇ ∷ []) "John.19.36"
∷ word (Ὀ ∷ σ ∷ τ ∷ ο ∷ ῦ ∷ ν ∷ []) "John.19.36"
∷ word (ο ∷ ὐ ∷ []) "John.19.36"
∷ word (σ ∷ υ ∷ ν ∷ τ ∷ ρ ∷ ι ∷ β ∷ ή ∷ σ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.19.36"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.19.36"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.19.37"
∷ word (π ∷ ά ∷ ∙λ ∷ ι ∷ ν ∷ []) "John.19.37"
∷ word (ἑ ∷ τ ∷ έ ∷ ρ ∷ α ∷ []) "John.19.37"
∷ word (γ ∷ ρ ∷ α ∷ φ ∷ ὴ ∷ []) "John.19.37"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.19.37"
∷ word (Ὄ ∷ ψ ∷ ο ∷ ν ∷ τ ∷ α ∷ ι ∷ []) "John.19.37"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.19.37"
∷ word (ὃ ∷ ν ∷ []) "John.19.37"
∷ word (ἐ ∷ ξ ∷ ε ∷ κ ∷ έ ∷ ν ∷ τ ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.19.37"
∷ word (Μ ∷ ε ∷ τ ∷ ὰ ∷ []) "John.19.38"
∷ word (δ ∷ ὲ ∷ []) "John.19.38"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.19.38"
∷ word (ἠ ∷ ρ ∷ ώ ∷ τ ∷ η ∷ σ ∷ ε ∷ ν ∷ []) "John.19.38"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.19.38"
∷ word (Π ∷ ι ∷ ∙λ ∷ ᾶ ∷ τ ∷ ο ∷ ν ∷ []) "John.19.38"
∷ word (Ἰ ∷ ω ∷ σ ∷ ὴ ∷ φ ∷ []) "John.19.38"
∷ word (ἀ ∷ π ∷ ὸ ∷ []) "John.19.38"
∷ word (Ἁ ∷ ρ ∷ ι ∷ μ ∷ α ∷ θ ∷ α ∷ ί ∷ α ∷ ς ∷ []) "John.19.38"
∷ word (ὢ ∷ ν ∷ []) "John.19.38"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ ὴ ∷ ς ∷ []) "John.19.38"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.19.38"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ []) "John.19.38"
∷ word (κ ∷ ε ∷ κ ∷ ρ ∷ υ ∷ μ ∷ μ ∷ έ ∷ ν ∷ ο ∷ ς ∷ []) "John.19.38"
∷ word (δ ∷ ὲ ∷ []) "John.19.38"
∷ word (δ ∷ ι ∷ ὰ ∷ []) "John.19.38"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.19.38"
∷ word (φ ∷ ό ∷ β ∷ ο ∷ ν ∷ []) "John.19.38"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.19.38"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ί ∷ ω ∷ ν ∷ []) "John.19.38"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.19.38"
∷ word (ἄ ∷ ρ ∷ ῃ ∷ []) "John.19.38"
∷ word (τ ∷ ὸ ∷ []) "John.19.38"
∷ word (σ ∷ ῶ ∷ μ ∷ α ∷ []) "John.19.38"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.19.38"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ []) "John.19.38"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.19.38"
∷ word (ἐ ∷ π ∷ έ ∷ τ ∷ ρ ∷ ε ∷ ψ ∷ ε ∷ ν ∷ []) "John.19.38"
∷ word (ὁ ∷ []) "John.19.38"
∷ word (Π ∷ ι ∷ ∙λ ∷ ᾶ ∷ τ ∷ ο ∷ ς ∷ []) "John.19.38"
∷ word (ἦ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.19.38"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.19.38"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.19.38"
∷ word (ἦ ∷ ρ ∷ ε ∷ ν ∷ []) "John.19.38"
∷ word (τ ∷ ὸ ∷ []) "John.19.38"
∷ word (σ ∷ ῶ ∷ μ ∷ α ∷ []) "John.19.38"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.19.38"
∷ word (ἦ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.19.39"
∷ word (δ ∷ ὲ ∷ []) "John.19.39"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.19.39"
∷ word (Ν ∷ ι ∷ κ ∷ ό ∷ δ ∷ η ∷ μ ∷ ο ∷ ς ∷ []) "John.19.39"
∷ word (ὁ ∷ []) "John.19.39"
∷ word (ἐ ∷ ∙λ ∷ θ ∷ ὼ ∷ ν ∷ []) "John.19.39"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.19.39"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.19.39"
∷ word (ν ∷ υ ∷ κ ∷ τ ∷ ὸ ∷ ς ∷ []) "John.19.39"
∷ word (τ ∷ ὸ ∷ []) "John.19.39"
∷ word (π ∷ ρ ∷ ῶ ∷ τ ∷ ο ∷ ν ∷ []) "John.19.39"
∷ word (φ ∷ έ ∷ ρ ∷ ω ∷ ν ∷ []) "John.19.39"
∷ word (μ ∷ ί ∷ γ ∷ μ ∷ α ∷ []) "John.19.39"
∷ word (σ ∷ μ ∷ ύ ∷ ρ ∷ ν ∷ η ∷ ς ∷ []) "John.19.39"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.19.39"
∷ word (ἀ ∷ ∙λ ∷ ό ∷ η ∷ ς ∷ []) "John.19.39"
∷ word (ὡ ∷ ς ∷ []) "John.19.39"
∷ word (∙λ ∷ ί ∷ τ ∷ ρ ∷ α ∷ ς ∷ []) "John.19.39"
∷ word (ἑ ∷ κ ∷ α ∷ τ ∷ ό ∷ ν ∷ []) "John.19.39"
∷ word (ἔ ∷ ∙λ ∷ α ∷ β ∷ ο ∷ ν ∷ []) "John.19.40"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.19.40"
∷ word (τ ∷ ὸ ∷ []) "John.19.40"
∷ word (σ ∷ ῶ ∷ μ ∷ α ∷ []) "John.19.40"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.19.40"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ []) "John.19.40"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.19.40"
∷ word (ἔ ∷ δ ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.19.40"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ []) "John.19.40"
∷ word (ὀ ∷ θ ∷ ο ∷ ν ∷ ί ∷ ο ∷ ι ∷ ς ∷ []) "John.19.40"
∷ word (μ ∷ ε ∷ τ ∷ ὰ ∷ []) "John.19.40"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.19.40"
∷ word (ἀ ∷ ρ ∷ ω ∷ μ ∷ ά ∷ τ ∷ ω ∷ ν ∷ []) "John.19.40"
∷ word (κ ∷ α ∷ θ ∷ ὼ ∷ ς ∷ []) "John.19.40"
∷ word (ἔ ∷ θ ∷ ο ∷ ς ∷ []) "John.19.40"
∷ word (ἐ ∷ σ ∷ τ ∷ ὶ ∷ ν ∷ []) "John.19.40"
∷ word (τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.19.40"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ί ∷ ο ∷ ι ∷ ς ∷ []) "John.19.40"
∷ word (ἐ ∷ ν ∷ τ ∷ α ∷ φ ∷ ι ∷ ά ∷ ζ ∷ ε ∷ ι ∷ ν ∷ []) "John.19.40"
∷ word (ἦ ∷ ν ∷ []) "John.19.41"
∷ word (δ ∷ ὲ ∷ []) "John.19.41"
∷ word (ἐ ∷ ν ∷ []) "John.19.41"
∷ word (τ ∷ ῷ ∷ []) "John.19.41"
∷ word (τ ∷ ό ∷ π ∷ ῳ ∷ []) "John.19.41"
∷ word (ὅ ∷ π ∷ ο ∷ υ ∷ []) "John.19.41"
∷ word (ἐ ∷ σ ∷ τ ∷ α ∷ υ ∷ ρ ∷ ώ ∷ θ ∷ η ∷ []) "John.19.41"
∷ word (κ ∷ ῆ ∷ π ∷ ο ∷ ς ∷ []) "John.19.41"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.19.41"
∷ word (ἐ ∷ ν ∷ []) "John.19.41"
∷ word (τ ∷ ῷ ∷ []) "John.19.41"
∷ word (κ ∷ ή ∷ π ∷ ῳ ∷ []) "John.19.41"
∷ word (μ ∷ ν ∷ η ∷ μ ∷ ε ∷ ῖ ∷ ο ∷ ν ∷ []) "John.19.41"
∷ word (κ ∷ α ∷ ι ∷ ν ∷ ό ∷ ν ∷ []) "John.19.41"
∷ word (ἐ ∷ ν ∷ []) "John.19.41"
∷ word (ᾧ ∷ []) "John.19.41"
∷ word (ο ∷ ὐ ∷ δ ∷ έ ∷ π ∷ ω ∷ []) "John.19.41"
∷ word (ο ∷ ὐ ∷ δ ∷ ε ∷ ὶ ∷ ς ∷ []) "John.19.41"
∷ word (ἦ ∷ ν ∷ []) "John.19.41"
∷ word (τ ∷ ε ∷ θ ∷ ε ∷ ι ∷ μ ∷ έ ∷ ν ∷ ο ∷ ς ∷ []) "John.19.41"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ []) "John.19.42"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.19.42"
∷ word (δ ∷ ι ∷ ὰ ∷ []) "John.19.42"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.19.42"
∷ word (π ∷ α ∷ ρ ∷ α ∷ σ ∷ κ ∷ ε ∷ υ ∷ ὴ ∷ ν ∷ []) "John.19.42"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.19.42"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ί ∷ ω ∷ ν ∷ []) "John.19.42"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.19.42"
∷ word (ἐ ∷ γ ∷ γ ∷ ὺ ∷ ς ∷ []) "John.19.42"
∷ word (ἦ ∷ ν ∷ []) "John.19.42"
∷ word (τ ∷ ὸ ∷ []) "John.19.42"
∷ word (μ ∷ ν ∷ η ∷ μ ∷ ε ∷ ῖ ∷ ο ∷ ν ∷ []) "John.19.42"
∷ word (ἔ ∷ θ ∷ η ∷ κ ∷ α ∷ ν ∷ []) "John.19.42"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.19.42"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ν ∷ []) "John.19.42"
∷ word (Τ ∷ ῇ ∷ []) "John.20.1"
∷ word (δ ∷ ὲ ∷ []) "John.20.1"
∷ word (μ ∷ ι ∷ ᾷ ∷ []) "John.20.1"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.20.1"
∷ word (σ ∷ α ∷ β ∷ β ∷ ά ∷ τ ∷ ω ∷ ν ∷ []) "John.20.1"
∷ word (Μ ∷ α ∷ ρ ∷ ί ∷ α ∷ []) "John.20.1"
∷ word (ἡ ∷ []) "John.20.1"
∷ word (Μ ∷ α ∷ γ ∷ δ ∷ α ∷ ∙λ ∷ η ∷ ν ∷ ὴ ∷ []) "John.20.1"
∷ word (ἔ ∷ ρ ∷ χ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.20.1"
∷ word (π ∷ ρ ∷ ω ∷ ῒ ∷ []) "John.20.1"
∷ word (σ ∷ κ ∷ ο ∷ τ ∷ ί ∷ α ∷ ς ∷ []) "John.20.1"
∷ word (ἔ ∷ τ ∷ ι ∷ []) "John.20.1"
∷ word (ο ∷ ὔ ∷ σ ∷ η ∷ ς ∷ []) "John.20.1"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.20.1"
∷ word (τ ∷ ὸ ∷ []) "John.20.1"
∷ word (μ ∷ ν ∷ η ∷ μ ∷ ε ∷ ῖ ∷ ο ∷ ν ∷ []) "John.20.1"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.1"
∷ word (β ∷ ∙λ ∷ έ ∷ π ∷ ε ∷ ι ∷ []) "John.20.1"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.20.1"
∷ word (∙λ ∷ ί ∷ θ ∷ ο ∷ ν ∷ []) "John.20.1"
∷ word (ἠ ∷ ρ ∷ μ ∷ έ ∷ ν ∷ ο ∷ ν ∷ []) "John.20.1"
∷ word (ἐ ∷ κ ∷ []) "John.20.1"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.20.1"
∷ word (μ ∷ ν ∷ η ∷ μ ∷ ε ∷ ί ∷ ο ∷ υ ∷ []) "John.20.1"
∷ word (τ ∷ ρ ∷ έ ∷ χ ∷ ε ∷ ι ∷ []) "John.20.2"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.20.2"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.2"
∷ word (ἔ ∷ ρ ∷ χ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.20.2"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.20.2"
∷ word (Σ ∷ ί ∷ μ ∷ ω ∷ ν ∷ α ∷ []) "John.20.2"
∷ word (Π ∷ έ ∷ τ ∷ ρ ∷ ο ∷ ν ∷ []) "John.20.2"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.2"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.20.2"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.20.2"
∷ word (ἄ ∷ ∙λ ∷ ∙λ ∷ ο ∷ ν ∷ []) "John.20.2"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ ὴ ∷ ν ∷ []) "John.20.2"
∷ word (ὃ ∷ ν ∷ []) "John.20.2"
∷ word (ἐ ∷ φ ∷ ί ∷ ∙λ ∷ ε ∷ ι ∷ []) "John.20.2"
∷ word (ὁ ∷ []) "John.20.2"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.20.2"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.2"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.20.2"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.20.2"
∷ word (Ἦ ∷ ρ ∷ α ∷ ν ∷ []) "John.20.2"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.20.2"
∷ word (κ ∷ ύ ∷ ρ ∷ ι ∷ ο ∷ ν ∷ []) "John.20.2"
∷ word (ἐ ∷ κ ∷ []) "John.20.2"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.20.2"
∷ word (μ ∷ ν ∷ η ∷ μ ∷ ε ∷ ί ∷ ο ∷ υ ∷ []) "John.20.2"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.2"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.20.2"
∷ word (ο ∷ ἴ ∷ δ ∷ α ∷ μ ∷ ε ∷ ν ∷ []) "John.20.2"
∷ word (π ∷ ο ∷ ῦ ∷ []) "John.20.2"
∷ word (ἔ ∷ θ ∷ η ∷ κ ∷ α ∷ ν ∷ []) "John.20.2"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.20.2"
∷ word (ἐ ∷ ξ ∷ ῆ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.20.3"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.20.3"
∷ word (ὁ ∷ []) "John.20.3"
∷ word (Π ∷ έ ∷ τ ∷ ρ ∷ ο ∷ ς ∷ []) "John.20.3"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.3"
∷ word (ὁ ∷ []) "John.20.3"
∷ word (ἄ ∷ ∙λ ∷ ∙λ ∷ ο ∷ ς ∷ []) "John.20.3"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ ή ∷ ς ∷ []) "John.20.3"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.3"
∷ word (ἤ ∷ ρ ∷ χ ∷ ο ∷ ν ∷ τ ∷ ο ∷ []) "John.20.3"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.20.3"
∷ word (τ ∷ ὸ ∷ []) "John.20.3"
∷ word (μ ∷ ν ∷ η ∷ μ ∷ ε ∷ ῖ ∷ ο ∷ ν ∷ []) "John.20.3"
∷ word (ἔ ∷ τ ∷ ρ ∷ ε ∷ χ ∷ ο ∷ ν ∷ []) "John.20.4"
∷ word (δ ∷ ὲ ∷ []) "John.20.4"
∷ word (ο ∷ ἱ ∷ []) "John.20.4"
∷ word (δ ∷ ύ ∷ ο ∷ []) "John.20.4"
∷ word (ὁ ∷ μ ∷ ο ∷ ῦ ∷ []) "John.20.4"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.4"
∷ word (ὁ ∷ []) "John.20.4"
∷ word (ἄ ∷ ∙λ ∷ ∙λ ∷ ο ∷ ς ∷ []) "John.20.4"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ ὴ ∷ ς ∷ []) "John.20.4"
∷ word (π ∷ ρ ∷ ο ∷ έ ∷ δ ∷ ρ ∷ α ∷ μ ∷ ε ∷ ν ∷ []) "John.20.4"
∷ word (τ ∷ ά ∷ χ ∷ ι ∷ ο ∷ ν ∷ []) "John.20.4"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.20.4"
∷ word (Π ∷ έ ∷ τ ∷ ρ ∷ ο ∷ υ ∷ []) "John.20.4"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.4"
∷ word (ἦ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.20.4"
∷ word (π ∷ ρ ∷ ῶ ∷ τ ∷ ο ∷ ς ∷ []) "John.20.4"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.20.4"
∷ word (τ ∷ ὸ ∷ []) "John.20.4"
∷ word (μ ∷ ν ∷ η ∷ μ ∷ ε ∷ ῖ ∷ ο ∷ ν ∷ []) "John.20.4"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.5"
∷ word (π ∷ α ∷ ρ ∷ α ∷ κ ∷ ύ ∷ ψ ∷ α ∷ ς ∷ []) "John.20.5"
∷ word (β ∷ ∙λ ∷ έ ∷ π ∷ ε ∷ ι ∷ []) "John.20.5"
∷ word (κ ∷ ε ∷ ί ∷ μ ∷ ε ∷ ν ∷ α ∷ []) "John.20.5"
∷ word (τ ∷ ὰ ∷ []) "John.20.5"
∷ word (ὀ ∷ θ ∷ ό ∷ ν ∷ ι ∷ α ∷ []) "John.20.5"
∷ word (ο ∷ ὐ ∷ []) "John.20.5"
∷ word (μ ∷ έ ∷ ν ∷ τ ∷ ο ∷ ι ∷ []) "John.20.5"
∷ word (ε ∷ ἰ ∷ σ ∷ ῆ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.20.5"
∷ word (ἔ ∷ ρ ∷ χ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.20.6"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.20.6"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.6"
∷ word (Σ ∷ ί ∷ μ ∷ ω ∷ ν ∷ []) "John.20.6"
∷ word (Π ∷ έ ∷ τ ∷ ρ ∷ ο ∷ ς ∷ []) "John.20.6"
∷ word (ἀ ∷ κ ∷ ο ∷ ∙λ ∷ ο ∷ υ ∷ θ ∷ ῶ ∷ ν ∷ []) "John.20.6"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.20.6"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.6"
∷ word (ε ∷ ἰ ∷ σ ∷ ῆ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.20.6"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.20.6"
∷ word (τ ∷ ὸ ∷ []) "John.20.6"
∷ word (μ ∷ ν ∷ η ∷ μ ∷ ε ∷ ῖ ∷ ο ∷ ν ∷ []) "John.20.6"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.6"
∷ word (θ ∷ ε ∷ ω ∷ ρ ∷ ε ∷ ῖ ∷ []) "John.20.6"
∷ word (τ ∷ ὰ ∷ []) "John.20.6"
∷ word (ὀ ∷ θ ∷ ό ∷ ν ∷ ι ∷ α ∷ []) "John.20.6"
∷ word (κ ∷ ε ∷ ί ∷ μ ∷ ε ∷ ν ∷ α ∷ []) "John.20.6"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.7"
∷ word (τ ∷ ὸ ∷ []) "John.20.7"
∷ word (σ ∷ ο ∷ υ ∷ δ ∷ ά ∷ ρ ∷ ι ∷ ο ∷ ν ∷ []) "John.20.7"
∷ word (ὃ ∷ []) "John.20.7"
∷ word (ἦ ∷ ν ∷ []) "John.20.7"
∷ word (ἐ ∷ π ∷ ὶ ∷ []) "John.20.7"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.20.7"
∷ word (κ ∷ ε ∷ φ ∷ α ∷ ∙λ ∷ ῆ ∷ ς ∷ []) "John.20.7"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.20.7"
∷ word (ο ∷ ὐ ∷ []) "John.20.7"
∷ word (μ ∷ ε ∷ τ ∷ ὰ ∷ []) "John.20.7"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.20.7"
∷ word (ὀ ∷ θ ∷ ο ∷ ν ∷ ί ∷ ω ∷ ν ∷ []) "John.20.7"
∷ word (κ ∷ ε ∷ ί ∷ μ ∷ ε ∷ ν ∷ ο ∷ ν ∷ []) "John.20.7"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.20.7"
∷ word (χ ∷ ω ∷ ρ ∷ ὶ ∷ ς ∷ []) "John.20.7"
∷ word (ἐ ∷ ν ∷ τ ∷ ε ∷ τ ∷ υ ∷ ∙λ ∷ ι ∷ γ ∷ μ ∷ έ ∷ ν ∷ ο ∷ ν ∷ []) "John.20.7"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.20.7"
∷ word (ἕ ∷ ν ∷ α ∷ []) "John.20.7"
∷ word (τ ∷ ό ∷ π ∷ ο ∷ ν ∷ []) "John.20.7"
∷ word (τ ∷ ό ∷ τ ∷ ε ∷ []) "John.20.8"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.20.8"
∷ word (ε ∷ ἰ ∷ σ ∷ ῆ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.20.8"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.8"
∷ word (ὁ ∷ []) "John.20.8"
∷ word (ἄ ∷ ∙λ ∷ ∙λ ∷ ο ∷ ς ∷ []) "John.20.8"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ ὴ ∷ ς ∷ []) "John.20.8"
∷ word (ὁ ∷ []) "John.20.8"
∷ word (ἐ ∷ ∙λ ∷ θ ∷ ὼ ∷ ν ∷ []) "John.20.8"
∷ word (π ∷ ρ ∷ ῶ ∷ τ ∷ ο ∷ ς ∷ []) "John.20.8"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.20.8"
∷ word (τ ∷ ὸ ∷ []) "John.20.8"
∷ word (μ ∷ ν ∷ η ∷ μ ∷ ε ∷ ῖ ∷ ο ∷ ν ∷ []) "John.20.8"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.8"
∷ word (ε ∷ ἶ ∷ δ ∷ ε ∷ ν ∷ []) "John.20.8"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.8"
∷ word (ἐ ∷ π ∷ ί ∷ σ ∷ τ ∷ ε ∷ υ ∷ σ ∷ ε ∷ ν ∷ []) "John.20.8"
∷ word (ο ∷ ὐ ∷ δ ∷ έ ∷ π ∷ ω ∷ []) "John.20.9"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.20.9"
∷ word (ᾔ ∷ δ ∷ ε ∷ ι ∷ σ ∷ α ∷ ν ∷ []) "John.20.9"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.20.9"
∷ word (γ ∷ ρ ∷ α ∷ φ ∷ ὴ ∷ ν ∷ []) "John.20.9"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.20.9"
∷ word (δ ∷ ε ∷ ῖ ∷ []) "John.20.9"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.20.9"
∷ word (ἐ ∷ κ ∷ []) "John.20.9"
∷ word (ν ∷ ε ∷ κ ∷ ρ ∷ ῶ ∷ ν ∷ []) "John.20.9"
∷ word (ἀ ∷ ν ∷ α ∷ σ ∷ τ ∷ ῆ ∷ ν ∷ α ∷ ι ∷ []) "John.20.9"
∷ word (ἀ ∷ π ∷ ῆ ∷ ∙λ ∷ θ ∷ ο ∷ ν ∷ []) "John.20.10"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.20.10"
∷ word (π ∷ ά ∷ ∙λ ∷ ι ∷ ν ∷ []) "John.20.10"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.20.10"
∷ word (α ∷ ὑ ∷ τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.20.10"
∷ word (ο ∷ ἱ ∷ []) "John.20.10"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ α ∷ ί ∷ []) "John.20.10"
∷ word (Μ ∷ α ∷ ρ ∷ ί ∷ α ∷ []) "John.20.11"
∷ word (δ ∷ ὲ ∷ []) "John.20.11"
∷ word (ε ∷ ἱ ∷ σ ∷ τ ∷ ή ∷ κ ∷ ε ∷ ι ∷ []) "John.20.11"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.20.11"
∷ word (τ ∷ ῷ ∷ []) "John.20.11"
∷ word (μ ∷ ν ∷ η ∷ μ ∷ ε ∷ ί ∷ ῳ ∷ []) "John.20.11"
∷ word (ἔ ∷ ξ ∷ ω ∷ []) "John.20.11"
∷ word (κ ∷ ∙λ ∷ α ∷ ί ∷ ο ∷ υ ∷ σ ∷ α ∷ []) "John.20.11"
∷ word (ὡ ∷ ς ∷ []) "John.20.11"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.20.11"
∷ word (ἔ ∷ κ ∷ ∙λ ∷ α ∷ ι ∷ ε ∷ ν ∷ []) "John.20.11"
∷ word (π ∷ α ∷ ρ ∷ έ ∷ κ ∷ υ ∷ ψ ∷ ε ∷ ν ∷ []) "John.20.11"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.20.11"
∷ word (τ ∷ ὸ ∷ []) "John.20.11"
∷ word (μ ∷ ν ∷ η ∷ μ ∷ ε ∷ ῖ ∷ ο ∷ ν ∷ []) "John.20.11"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.12"
∷ word (θ ∷ ε ∷ ω ∷ ρ ∷ ε ∷ ῖ ∷ []) "John.20.12"
∷ word (δ ∷ ύ ∷ ο ∷ []) "John.20.12"
∷ word (ἀ ∷ γ ∷ γ ∷ έ ∷ ∙λ ∷ ο ∷ υ ∷ ς ∷ []) "John.20.12"
∷ word (ἐ ∷ ν ∷ []) "John.20.12"
∷ word (∙λ ∷ ε ∷ υ ∷ κ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.20.12"
∷ word (κ ∷ α ∷ θ ∷ ε ∷ ζ ∷ ο ∷ μ ∷ έ ∷ ν ∷ ο ∷ υ ∷ ς ∷ []) "John.20.12"
∷ word (ἕ ∷ ν ∷ α ∷ []) "John.20.12"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.20.12"
∷ word (τ ∷ ῇ ∷ []) "John.20.12"
∷ word (κ ∷ ε ∷ φ ∷ α ∷ ∙λ ∷ ῇ ∷ []) "John.20.12"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.12"
∷ word (ἕ ∷ ν ∷ α ∷ []) "John.20.12"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.20.12"
∷ word (τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.20.12"
∷ word (π ∷ ο ∷ σ ∷ ί ∷ ν ∷ []) "John.20.12"
∷ word (ὅ ∷ π ∷ ο ∷ υ ∷ []) "John.20.12"
∷ word (ἔ ∷ κ ∷ ε ∷ ι ∷ τ ∷ ο ∷ []) "John.20.12"
∷ word (τ ∷ ὸ ∷ []) "John.20.12"
∷ word (σ ∷ ῶ ∷ μ ∷ α ∷ []) "John.20.12"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.20.12"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ []) "John.20.12"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.13"
∷ word (∙λ ∷ έ ∷ γ ∷ ο ∷ υ ∷ σ ∷ ι ∷ ν ∷ []) "John.20.13"
∷ word (α ∷ ὐ ∷ τ ∷ ῇ ∷ []) "John.20.13"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ο ∷ ι ∷ []) "John.20.13"
∷ word (Γ ∷ ύ ∷ ν ∷ α ∷ ι ∷ []) "John.20.13"
∷ word (τ ∷ ί ∷ []) "John.20.13"
∷ word (κ ∷ ∙λ ∷ α ∷ ί ∷ ε ∷ ι ∷ ς ∷ []) "John.20.13"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.20.13"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.20.13"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.20.13"
∷ word (Ἦ ∷ ρ ∷ α ∷ ν ∷ []) "John.20.13"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.20.13"
∷ word (κ ∷ ύ ∷ ρ ∷ ι ∷ ό ∷ ν ∷ []) "John.20.13"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.20.13"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.13"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.20.13"
∷ word (ο ∷ ἶ ∷ δ ∷ α ∷ []) "John.20.13"
∷ word (π ∷ ο ∷ ῦ ∷ []) "John.20.13"
∷ word (ἔ ∷ θ ∷ η ∷ κ ∷ α ∷ ν ∷ []) "John.20.13"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.20.13"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.20.14"
∷ word (ε ∷ ἰ ∷ π ∷ ο ∷ ῦ ∷ σ ∷ α ∷ []) "John.20.14"
∷ word (ἐ ∷ σ ∷ τ ∷ ρ ∷ ά ∷ φ ∷ η ∷ []) "John.20.14"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.20.14"
∷ word (τ ∷ ὰ ∷ []) "John.20.14"
∷ word (ὀ ∷ π ∷ ί ∷ σ ∷ ω ∷ []) "John.20.14"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.14"
∷ word (θ ∷ ε ∷ ω ∷ ρ ∷ ε ∷ ῖ ∷ []) "John.20.14"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.20.14"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ν ∷ []) "John.20.14"
∷ word (ἑ ∷ σ ∷ τ ∷ ῶ ∷ τ ∷ α ∷ []) "John.20.14"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.14"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.20.14"
∷ word (ᾔ ∷ δ ∷ ε ∷ ι ∷ []) "John.20.14"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.20.14"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.20.14"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.20.14"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.20.15"
∷ word (α ∷ ὐ ∷ τ ∷ ῇ ∷ []) "John.20.15"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.20.15"
∷ word (Γ ∷ ύ ∷ ν ∷ α ∷ ι ∷ []) "John.20.15"
∷ word (τ ∷ ί ∷ []) "John.20.15"
∷ word (κ ∷ ∙λ ∷ α ∷ ί ∷ ε ∷ ι ∷ ς ∷ []) "John.20.15"
∷ word (τ ∷ ί ∷ ν ∷ α ∷ []) "John.20.15"
∷ word (ζ ∷ η ∷ τ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.20.15"
∷ word (ἐ ∷ κ ∷ ε ∷ ί ∷ ν ∷ η ∷ []) "John.20.15"
∷ word (δ ∷ ο ∷ κ ∷ ο ∷ ῦ ∷ σ ∷ α ∷ []) "John.20.15"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.20.15"
∷ word (ὁ ∷ []) "John.20.15"
∷ word (κ ∷ η ∷ π ∷ ο ∷ υ ∷ ρ ∷ ό ∷ ς ∷ []) "John.20.15"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.20.15"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.20.15"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.20.15"
∷ word (Κ ∷ ύ ∷ ρ ∷ ι ∷ ε ∷ []) "John.20.15"
∷ word (ε ∷ ἰ ∷ []) "John.20.15"
∷ word (σ ∷ ὺ ∷ []) "John.20.15"
∷ word (ἐ ∷ β ∷ ά ∷ σ ∷ τ ∷ α ∷ σ ∷ α ∷ ς ∷ []) "John.20.15"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.20.15"
∷ word (ε ∷ ἰ ∷ π ∷ έ ∷ []) "John.20.15"
∷ word (μ ∷ ο ∷ ι ∷ []) "John.20.15"
∷ word (π ∷ ο ∷ ῦ ∷ []) "John.20.15"
∷ word (ἔ ∷ θ ∷ η ∷ κ ∷ α ∷ ς ∷ []) "John.20.15"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.20.15"
∷ word (κ ∷ ἀ ∷ γ ∷ ὼ ∷ []) "John.20.15"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.20.15"
∷ word (ἀ ∷ ρ ∷ ῶ ∷ []) "John.20.15"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.20.16"
∷ word (α ∷ ὐ ∷ τ ∷ ῇ ∷ []) "John.20.16"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.20.16"
∷ word (Μ ∷ α ∷ ρ ∷ ι ∷ ά ∷ μ ∷ []) "John.20.16"
∷ word (σ ∷ τ ∷ ρ ∷ α ∷ φ ∷ ε ∷ ῖ ∷ σ ∷ α ∷ []) "John.20.16"
∷ word (ἐ ∷ κ ∷ ε ∷ ί ∷ ν ∷ η ∷ []) "John.20.16"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.20.16"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.20.16"
∷ word (Ἑ ∷ β ∷ ρ ∷ α ∷ ϊ ∷ σ ∷ τ ∷ ί ∷ []) "John.20.16"
∷ word (Ρ ∷ α ∷ β ∷ β ∷ ο ∷ υ ∷ ν ∷ ι ∷ []) "John.20.16"
∷ word (ὃ ∷ []) "John.20.16"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.20.16"
∷ word (Δ ∷ ι ∷ δ ∷ ά ∷ σ ∷ κ ∷ α ∷ ∙λ ∷ ε ∷ []) "John.20.16"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.20.17"
∷ word (α ∷ ὐ ∷ τ ∷ ῇ ∷ []) "John.20.17"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.20.17"
∷ word (Μ ∷ ή ∷ []) "John.20.17"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.20.17"
∷ word (ἅ ∷ π ∷ τ ∷ ο ∷ υ ∷ []) "John.20.17"
∷ word (ο ∷ ὔ ∷ π ∷ ω ∷ []) "John.20.17"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.20.17"
∷ word (ἀ ∷ ν ∷ α ∷ β ∷ έ ∷ β ∷ η ∷ κ ∷ α ∷ []) "John.20.17"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.20.17"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.20.17"
∷ word (π ∷ α ∷ τ ∷ έ ∷ ρ ∷ α ∷ []) "John.20.17"
∷ word (π ∷ ο ∷ ρ ∷ ε ∷ ύ ∷ ο ∷ υ ∷ []) "John.20.17"
∷ word (δ ∷ ὲ ∷ []) "John.20.17"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.20.17"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.20.17"
∷ word (ἀ ∷ δ ∷ ε ∷ ∙λ ∷ φ ∷ ο ∷ ύ ∷ ς ∷ []) "John.20.17"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.20.17"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.17"
∷ word (ε ∷ ἰ ∷ π ∷ ὲ ∷ []) "John.20.17"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.20.17"
∷ word (Ἀ ∷ ν ∷ α ∷ β ∷ α ∷ ί ∷ ν ∷ ω ∷ []) "John.20.17"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.20.17"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.20.17"
∷ word (π ∷ α ∷ τ ∷ έ ∷ ρ ∷ α ∷ []) "John.20.17"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.20.17"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.17"
∷ word (π ∷ α ∷ τ ∷ έ ∷ ρ ∷ α ∷ []) "John.20.17"
∷ word (ὑ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.20.17"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.17"
∷ word (θ ∷ ε ∷ ό ∷ ν ∷ []) "John.20.17"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.20.17"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.17"
∷ word (θ ∷ ε ∷ ὸ ∷ ν ∷ []) "John.20.17"
∷ word (ὑ ∷ μ ∷ ῶ ∷ ν ∷ []) "John.20.17"
∷ word (ἔ ∷ ρ ∷ χ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.20.18"
∷ word (Μ ∷ α ∷ ρ ∷ ι ∷ ὰ ∷ μ ∷ []) "John.20.18"
∷ word (ἡ ∷ []) "John.20.18"
∷ word (Μ ∷ α ∷ γ ∷ δ ∷ α ∷ ∙λ ∷ η ∷ ν ∷ ὴ ∷ []) "John.20.18"
∷ word (ἀ ∷ γ ∷ γ ∷ έ ∷ ∙λ ∷ ∙λ ∷ ο ∷ υ ∷ σ ∷ α ∷ []) "John.20.18"
∷ word (τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.20.18"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ α ∷ ῖ ∷ ς ∷ []) "John.20.18"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.20.18"
∷ word (Ἑ ∷ ώ ∷ ρ ∷ α ∷ κ ∷ α ∷ []) "John.20.18"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.20.18"
∷ word (κ ∷ ύ ∷ ρ ∷ ι ∷ ο ∷ ν ∷ []) "John.20.18"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.18"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.20.18"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.20.18"
∷ word (α ∷ ὐ ∷ τ ∷ ῇ ∷ []) "John.20.18"
∷ word (Ο ∷ ὔ ∷ σ ∷ η ∷ ς ∷ []) "John.20.19"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.20.19"
∷ word (ὀ ∷ ψ ∷ ί ∷ α ∷ ς ∷ []) "John.20.19"
∷ word (τ ∷ ῇ ∷ []) "John.20.19"
∷ word (ἡ ∷ μ ∷ έ ∷ ρ ∷ ᾳ ∷ []) "John.20.19"
∷ word (ἐ ∷ κ ∷ ε ∷ ί ∷ ν ∷ ῃ ∷ []) "John.20.19"
∷ word (τ ∷ ῇ ∷ []) "John.20.19"
∷ word (μ ∷ ι ∷ ᾷ ∷ []) "John.20.19"
∷ word (σ ∷ α ∷ β ∷ β ∷ ά ∷ τ ∷ ω ∷ ν ∷ []) "John.20.19"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.19"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.20.19"
∷ word (θ ∷ υ ∷ ρ ∷ ῶ ∷ ν ∷ []) "John.20.19"
∷ word (κ ∷ ε ∷ κ ∷ ∙λ ∷ ε ∷ ι ∷ σ ∷ μ ∷ έ ∷ ν ∷ ω ∷ ν ∷ []) "John.20.19"
∷ word (ὅ ∷ π ∷ ο ∷ υ ∷ []) "John.20.19"
∷ word (ἦ ∷ σ ∷ α ∷ ν ∷ []) "John.20.19"
∷ word (ο ∷ ἱ ∷ []) "John.20.19"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ α ∷ ὶ ∷ []) "John.20.19"
∷ word (δ ∷ ι ∷ ὰ ∷ []) "John.20.19"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.20.19"
∷ word (φ ∷ ό ∷ β ∷ ο ∷ ν ∷ []) "John.20.19"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.20.19"
∷ word (Ἰ ∷ ο ∷ υ ∷ δ ∷ α ∷ ί ∷ ω ∷ ν ∷ []) "John.20.19"
∷ word (ἦ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.20.19"
∷ word (ὁ ∷ []) "John.20.19"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.20.19"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.19"
∷ word (ἔ ∷ σ ∷ τ ∷ η ∷ []) "John.20.19"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.20.19"
∷ word (τ ∷ ὸ ∷ []) "John.20.19"
∷ word (μ ∷ έ ∷ σ ∷ ο ∷ ν ∷ []) "John.20.19"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.19"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.20.19"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.20.19"
∷ word (Ε ∷ ἰ ∷ ρ ∷ ή ∷ ν ∷ η ∷ []) "John.20.19"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.20.19"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.20"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.20.20"
∷ word (ε ∷ ἰ ∷ π ∷ ὼ ∷ ν ∷ []) "John.20.20"
∷ word (ἔ ∷ δ ∷ ε ∷ ι ∷ ξ ∷ ε ∷ ν ∷ []) "John.20.20"
∷ word (τ ∷ ὰ ∷ ς ∷ []) "John.20.20"
∷ word (χ ∷ ε ∷ ῖ ∷ ρ ∷ α ∷ ς ∷ []) "John.20.20"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.20"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.20.20"
∷ word (π ∷ ∙λ ∷ ε ∷ υ ∷ ρ ∷ ὰ ∷ ν ∷ []) "John.20.20"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.20.20"
∷ word (ἐ ∷ χ ∷ ά ∷ ρ ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.20.20"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.20.20"
∷ word (ο ∷ ἱ ∷ []) "John.20.20"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ α ∷ ὶ ∷ []) "John.20.20"
∷ word (ἰ ∷ δ ∷ ό ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.20.20"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.20.20"
∷ word (κ ∷ ύ ∷ ρ ∷ ι ∷ ο ∷ ν ∷ []) "John.20.20"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.20.21"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.20.21"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.20.21"
∷ word (ὁ ∷ []) "John.20.21"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.20.21"
∷ word (π ∷ ά ∷ ∙λ ∷ ι ∷ ν ∷ []) "John.20.21"
∷ word (Ε ∷ ἰ ∷ ρ ∷ ή ∷ ν ∷ η ∷ []) "John.20.21"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.20.21"
∷ word (κ ∷ α ∷ θ ∷ ὼ ∷ ς ∷ []) "John.20.21"
∷ word (ἀ ∷ π ∷ έ ∷ σ ∷ τ ∷ α ∷ ∙λ ∷ κ ∷ έ ∷ ν ∷ []) "John.20.21"
∷ word (μ ∷ ε ∷ []) "John.20.21"
∷ word (ὁ ∷ []) "John.20.21"
∷ word (π ∷ α ∷ τ ∷ ή ∷ ρ ∷ []) "John.20.21"
∷ word (κ ∷ ἀ ∷ γ ∷ ὼ ∷ []) "John.20.21"
∷ word (π ∷ έ ∷ μ ∷ π ∷ ω ∷ []) "John.20.21"
∷ word (ὑ ∷ μ ∷ ᾶ ∷ ς ∷ []) "John.20.21"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.22"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.20.22"
∷ word (ε ∷ ἰ ∷ π ∷ ὼ ∷ ν ∷ []) "John.20.22"
∷ word (ἐ ∷ ν ∷ ε ∷ φ ∷ ύ ∷ σ ∷ η ∷ σ ∷ ε ∷ ν ∷ []) "John.20.22"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.22"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.20.22"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.20.22"
∷ word (Λ ∷ ά ∷ β ∷ ε ∷ τ ∷ ε ∷ []) "John.20.22"
∷ word (π ∷ ν ∷ ε ∷ ῦ ∷ μ ∷ α ∷ []) "John.20.22"
∷ word (ἅ ∷ γ ∷ ι ∷ ο ∷ ν ∷ []) "John.20.22"
∷ word (ἄ ∷ ν ∷ []) "John.20.23"
∷ word (τ ∷ ι ∷ ν ∷ ω ∷ ν ∷ []) "John.20.23"
∷ word (ἀ ∷ φ ∷ ῆ ∷ τ ∷ ε ∷ []) "John.20.23"
∷ word (τ ∷ ὰ ∷ ς ∷ []) "John.20.23"
∷ word (ἁ ∷ μ ∷ α ∷ ρ ∷ τ ∷ ί ∷ α ∷ ς ∷ []) "John.20.23"
∷ word (ἀ ∷ φ ∷ έ ∷ ω ∷ ν ∷ τ ∷ α ∷ ι ∷ []) "John.20.23"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.20.23"
∷ word (ἄ ∷ ν ∷ []) "John.20.23"
∷ word (τ ∷ ι ∷ ν ∷ ω ∷ ν ∷ []) "John.20.23"
∷ word (κ ∷ ρ ∷ α ∷ τ ∷ ῆ ∷ τ ∷ ε ∷ []) "John.20.23"
∷ word (κ ∷ ε ∷ κ ∷ ρ ∷ ά ∷ τ ∷ η ∷ ν ∷ τ ∷ α ∷ ι ∷ []) "John.20.23"
∷ word (Θ ∷ ω ∷ μ ∷ ᾶ ∷ ς ∷ []) "John.20.24"
∷ word (δ ∷ ὲ ∷ []) "John.20.24"
∷ word (ε ∷ ἷ ∷ ς ∷ []) "John.20.24"
∷ word (ἐ ∷ κ ∷ []) "John.20.24"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.20.24"
∷ word (δ ∷ ώ ∷ δ ∷ ε ∷ κ ∷ α ∷ []) "John.20.24"
∷ word (ὁ ∷ []) "John.20.24"
∷ word (∙λ ∷ ε ∷ γ ∷ ό ∷ μ ∷ ε ∷ ν ∷ ο ∷ ς ∷ []) "John.20.24"
∷ word (Δ ∷ ί ∷ δ ∷ υ ∷ μ ∷ ο ∷ ς ∷ []) "John.20.24"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.20.24"
∷ word (ἦ ∷ ν ∷ []) "John.20.24"
∷ word (μ ∷ ε ∷ τ ∷ []) "John.20.24"
∷ word (α ∷ ὐ ∷ τ ∷ ῶ ∷ ν ∷ []) "John.20.24"
∷ word (ὅ ∷ τ ∷ ε ∷ []) "John.20.24"
∷ word (ἦ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.20.24"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.20.24"
∷ word (ἔ ∷ ∙λ ∷ ε ∷ γ ∷ ο ∷ ν ∷ []) "John.20.25"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.20.25"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.20.25"
∷ word (ο ∷ ἱ ∷ []) "John.20.25"
∷ word (ἄ ∷ ∙λ ∷ ∙λ ∷ ο ∷ ι ∷ []) "John.20.25"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ α ∷ ί ∷ []) "John.20.25"
∷ word (Ἑ ∷ ω ∷ ρ ∷ ά ∷ κ ∷ α ∷ μ ∷ ε ∷ ν ∷ []) "John.20.25"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.20.25"
∷ word (κ ∷ ύ ∷ ρ ∷ ι ∷ ο ∷ ν ∷ []) "John.20.25"
∷ word (ὁ ∷ []) "John.20.25"
∷ word (δ ∷ ὲ ∷ []) "John.20.25"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.20.25"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.20.25"
∷ word (Ἐ ∷ ὰ ∷ ν ∷ []) "John.20.25"
∷ word (μ ∷ ὴ ∷ []) "John.20.25"
∷ word (ἴ ∷ δ ∷ ω ∷ []) "John.20.25"
∷ word (ἐ ∷ ν ∷ []) "John.20.25"
∷ word (τ ∷ α ∷ ῖ ∷ ς ∷ []) "John.20.25"
∷ word (χ ∷ ε ∷ ρ ∷ σ ∷ ὶ ∷ ν ∷ []) "John.20.25"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.20.25"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.20.25"
∷ word (τ ∷ ύ ∷ π ∷ ο ∷ ν ∷ []) "John.20.25"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.20.25"
∷ word (ἥ ∷ ∙λ ∷ ω ∷ ν ∷ []) "John.20.25"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.25"
∷ word (β ∷ ά ∷ ∙λ ∷ ω ∷ []) "John.20.25"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.20.25"
∷ word (δ ∷ ά ∷ κ ∷ τ ∷ υ ∷ ∙λ ∷ ό ∷ ν ∷ []) "John.20.25"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.20.25"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.20.25"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.20.25"
∷ word (τ ∷ ύ ∷ π ∷ ο ∷ ν ∷ []) "John.20.25"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.20.25"
∷ word (ἥ ∷ ∙λ ∷ ω ∷ ν ∷ []) "John.20.25"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.25"
∷ word (β ∷ ά ∷ ∙λ ∷ ω ∷ []) "John.20.25"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.20.25"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.20.25"
∷ word (χ ∷ ε ∷ ῖ ∷ ρ ∷ α ∷ []) "John.20.25"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.20.25"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.20.25"
∷ word (π ∷ ∙λ ∷ ε ∷ υ ∷ ρ ∷ ὰ ∷ ν ∷ []) "John.20.25"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.20.25"
∷ word (ο ∷ ὐ ∷ []) "John.20.25"
∷ word (μ ∷ ὴ ∷ []) "John.20.25"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ σ ∷ ω ∷ []) "John.20.25"
∷ word (Κ ∷ α ∷ ὶ ∷ []) "John.20.26"
∷ word (μ ∷ ε ∷ θ ∷ []) "John.20.26"
∷ word (ἡ ∷ μ ∷ έ ∷ ρ ∷ α ∷ ς ∷ []) "John.20.26"
∷ word (ὀ ∷ κ ∷ τ ∷ ὼ ∷ []) "John.20.26"
∷ word (π ∷ ά ∷ ∙λ ∷ ι ∷ ν ∷ []) "John.20.26"
∷ word (ἦ ∷ σ ∷ α ∷ ν ∷ []) "John.20.26"
∷ word (ἔ ∷ σ ∷ ω ∷ []) "John.20.26"
∷ word (ο ∷ ἱ ∷ []) "John.20.26"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ α ∷ ὶ ∷ []) "John.20.26"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.20.26"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.26"
∷ word (Θ ∷ ω ∷ μ ∷ ᾶ ∷ ς ∷ []) "John.20.26"
∷ word (μ ∷ ε ∷ τ ∷ []) "John.20.26"
∷ word (α ∷ ὐ ∷ τ ∷ ῶ ∷ ν ∷ []) "John.20.26"
∷ word (ἔ ∷ ρ ∷ χ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.20.26"
∷ word (ὁ ∷ []) "John.20.26"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.20.26"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.20.26"
∷ word (θ ∷ υ ∷ ρ ∷ ῶ ∷ ν ∷ []) "John.20.26"
∷ word (κ ∷ ε ∷ κ ∷ ∙λ ∷ ε ∷ ι ∷ σ ∷ μ ∷ έ ∷ ν ∷ ω ∷ ν ∷ []) "John.20.26"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.26"
∷ word (ἔ ∷ σ ∷ τ ∷ η ∷ []) "John.20.26"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.20.26"
∷ word (τ ∷ ὸ ∷ []) "John.20.26"
∷ word (μ ∷ έ ∷ σ ∷ ο ∷ ν ∷ []) "John.20.26"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.26"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.20.26"
∷ word (Ε ∷ ἰ ∷ ρ ∷ ή ∷ ν ∷ η ∷ []) "John.20.26"
∷ word (ὑ ∷ μ ∷ ῖ ∷ ν ∷ []) "John.20.26"
∷ word (ε ∷ ἶ ∷ τ ∷ α ∷ []) "John.20.27"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.20.27"
∷ word (τ ∷ ῷ ∷ []) "John.20.27"
∷ word (Θ ∷ ω ∷ μ ∷ ᾷ ∷ []) "John.20.27"
∷ word (Φ ∷ έ ∷ ρ ∷ ε ∷ []) "John.20.27"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.20.27"
∷ word (δ ∷ ά ∷ κ ∷ τ ∷ υ ∷ ∙λ ∷ ό ∷ ν ∷ []) "John.20.27"
∷ word (σ ∷ ο ∷ υ ∷ []) "John.20.27"
∷ word (ὧ ∷ δ ∷ ε ∷ []) "John.20.27"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.27"
∷ word (ἴ ∷ δ ∷ ε ∷ []) "John.20.27"
∷ word (τ ∷ ὰ ∷ ς ∷ []) "John.20.27"
∷ word (χ ∷ ε ∷ ῖ ∷ ρ ∷ ά ∷ ς ∷ []) "John.20.27"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.20.27"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.27"
∷ word (φ ∷ έ ∷ ρ ∷ ε ∷ []) "John.20.27"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.20.27"
∷ word (χ ∷ ε ∷ ῖ ∷ ρ ∷ ά ∷ []) "John.20.27"
∷ word (σ ∷ ο ∷ υ ∷ []) "John.20.27"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.27"
∷ word (β ∷ ά ∷ ∙λ ∷ ε ∷ []) "John.20.27"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.20.27"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.20.27"
∷ word (π ∷ ∙λ ∷ ε ∷ υ ∷ ρ ∷ ά ∷ ν ∷ []) "John.20.27"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.20.27"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.27"
∷ word (μ ∷ ὴ ∷ []) "John.20.27"
∷ word (γ ∷ ί ∷ ν ∷ ο ∷ υ ∷ []) "John.20.27"
∷ word (ἄ ∷ π ∷ ι ∷ σ ∷ τ ∷ ο ∷ ς ∷ []) "John.20.27"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.20.27"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ό ∷ ς ∷ []) "John.20.27"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ []) "John.20.28"
∷ word (Θ ∷ ω ∷ μ ∷ ᾶ ∷ ς ∷ []) "John.20.28"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.28"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.20.28"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.20.28"
∷ word (Ὁ ∷ []) "John.20.28"
∷ word (κ ∷ ύ ∷ ρ ∷ ι ∷ ό ∷ ς ∷ []) "John.20.28"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.20.28"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.28"
∷ word (ὁ ∷ []) "John.20.28"
∷ word (θ ∷ ε ∷ ό ∷ ς ∷ []) "John.20.28"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.20.28"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.20.29"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.20.29"
∷ word (ὁ ∷ []) "John.20.29"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.20.29"
∷ word (Ὅ ∷ τ ∷ ι ∷ []) "John.20.29"
∷ word (ἑ ∷ ώ ∷ ρ ∷ α ∷ κ ∷ ά ∷ ς ∷ []) "John.20.29"
∷ word (μ ∷ ε ∷ []) "John.20.29"
∷ word (π ∷ ε ∷ π ∷ ί ∷ σ ∷ τ ∷ ε ∷ υ ∷ κ ∷ α ∷ ς ∷ []) "John.20.29"
∷ word (μ ∷ α ∷ κ ∷ ά ∷ ρ ∷ ι ∷ ο ∷ ι ∷ []) "John.20.29"
∷ word (ο ∷ ἱ ∷ []) "John.20.29"
∷ word (μ ∷ ὴ ∷ []) "John.20.29"
∷ word (ἰ ∷ δ ∷ ό ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.20.29"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.29"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ σ ∷ α ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.20.29"
∷ word (Π ∷ ο ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.20.30"
∷ word (μ ∷ ὲ ∷ ν ∷ []) "John.20.30"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.20.30"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.30"
∷ word (ἄ ∷ ∙λ ∷ ∙λ ∷ α ∷ []) "John.20.30"
∷ word (σ ∷ η ∷ μ ∷ ε ∷ ῖ ∷ α ∷ []) "John.20.30"
∷ word (ἐ ∷ π ∷ ο ∷ ί ∷ η ∷ σ ∷ ε ∷ ν ∷ []) "John.20.30"
∷ word (ὁ ∷ []) "John.20.30"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.20.30"
∷ word (ἐ ∷ ν ∷ ώ ∷ π ∷ ι ∷ ο ∷ ν ∷ []) "John.20.30"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.20.30"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ ῶ ∷ ν ∷ []) "John.20.30"
∷ word (ἃ ∷ []) "John.20.30"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.20.30"
∷ word (ἔ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.20.30"
∷ word (γ ∷ ε ∷ γ ∷ ρ ∷ α ∷ μ ∷ μ ∷ έ ∷ ν ∷ α ∷ []) "John.20.30"
∷ word (ἐ ∷ ν ∷ []) "John.20.30"
∷ word (τ ∷ ῷ ∷ []) "John.20.30"
∷ word (β ∷ ι ∷ β ∷ ∙λ ∷ ί ∷ ῳ ∷ []) "John.20.30"
∷ word (τ ∷ ο ∷ ύ ∷ τ ∷ ῳ ∷ []) "John.20.30"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.20.31"
∷ word (δ ∷ ὲ ∷ []) "John.20.31"
∷ word (γ ∷ έ ∷ γ ∷ ρ ∷ α ∷ π ∷ τ ∷ α ∷ ι ∷ []) "John.20.31"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.20.31"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ η ∷ τ ∷ ε ∷ []) "John.20.31"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.20.31"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.20.31"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.20.31"
∷ word (ὁ ∷ []) "John.20.31"
∷ word (χ ∷ ρ ∷ ι ∷ σ ∷ τ ∷ ὸ ∷ ς ∷ []) "John.20.31"
∷ word (ὁ ∷ []) "John.20.31"
∷ word (υ ∷ ἱ ∷ ὸ ∷ ς ∷ []) "John.20.31"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.20.31"
∷ word (θ ∷ ε ∷ ο ∷ ῦ ∷ []) "John.20.31"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.20.31"
∷ word (ἵ ∷ ν ∷ α ∷ []) "John.20.31"
∷ word (π ∷ ι ∷ σ ∷ τ ∷ ε ∷ ύ ∷ ο ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.20.31"
∷ word (ζ ∷ ω ∷ ὴ ∷ ν ∷ []) "John.20.31"
∷ word (ἔ ∷ χ ∷ η ∷ τ ∷ ε ∷ []) "John.20.31"
∷ word (ἐ ∷ ν ∷ []) "John.20.31"
∷ word (τ ∷ ῷ ∷ []) "John.20.31"
∷ word (ὀ ∷ ν ∷ ό ∷ μ ∷ α ∷ τ ∷ ι ∷ []) "John.20.31"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.20.31"
∷ word (Μ ∷ ε ∷ τ ∷ ὰ ∷ []) "John.21.1"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.21.1"
∷ word (ἐ ∷ φ ∷ α ∷ ν ∷ έ ∷ ρ ∷ ω ∷ σ ∷ ε ∷ ν ∷ []) "John.21.1"
∷ word (ἑ ∷ α ∷ υ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.21.1"
∷ word (π ∷ ά ∷ ∙λ ∷ ι ∷ ν ∷ []) "John.21.1"
∷ word (ὁ ∷ []) "John.21.1"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.21.1"
∷ word (τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.21.1"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ α ∷ ῖ ∷ ς ∷ []) "John.21.1"
∷ word (ἐ ∷ π ∷ ὶ ∷ []) "John.21.1"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.21.1"
∷ word (θ ∷ α ∷ ∙λ ∷ ά ∷ σ ∷ σ ∷ η ∷ ς ∷ []) "John.21.1"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.21.1"
∷ word (Τ ∷ ι ∷ β ∷ ε ∷ ρ ∷ ι ∷ ά ∷ δ ∷ ο ∷ ς ∷ []) "John.21.1"
∷ word (ἐ ∷ φ ∷ α ∷ ν ∷ έ ∷ ρ ∷ ω ∷ σ ∷ ε ∷ ν ∷ []) "John.21.1"
∷ word (δ ∷ ὲ ∷ []) "John.21.1"
∷ word (ο ∷ ὕ ∷ τ ∷ ω ∷ ς ∷ []) "John.21.1"
∷ word (ἦ ∷ σ ∷ α ∷ ν ∷ []) "John.21.2"
∷ word (ὁ ∷ μ ∷ ο ∷ ῦ ∷ []) "John.21.2"
∷ word (Σ ∷ ί ∷ μ ∷ ω ∷ ν ∷ []) "John.21.2"
∷ word (Π ∷ έ ∷ τ ∷ ρ ∷ ο ∷ ς ∷ []) "John.21.2"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.21.2"
∷ word (Θ ∷ ω ∷ μ ∷ ᾶ ∷ ς ∷ []) "John.21.2"
∷ word (ὁ ∷ []) "John.21.2"
∷ word (∙λ ∷ ε ∷ γ ∷ ό ∷ μ ∷ ε ∷ ν ∷ ο ∷ ς ∷ []) "John.21.2"
∷ word (Δ ∷ ί ∷ δ ∷ υ ∷ μ ∷ ο ∷ ς ∷ []) "John.21.2"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.21.2"
∷ word (Ν ∷ α ∷ θ ∷ α ∷ ν ∷ α ∷ ὴ ∷ ∙λ ∷ []) "John.21.2"
∷ word (ὁ ∷ []) "John.21.2"
∷ word (ἀ ∷ π ∷ ὸ ∷ []) "John.21.2"
∷ word (Κ ∷ α ∷ ν ∷ ὰ ∷ []) "John.21.2"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.21.2"
∷ word (Γ ∷ α ∷ ∙λ ∷ ι ∷ ∙λ ∷ α ∷ ί ∷ α ∷ ς ∷ []) "John.21.2"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.21.2"
∷ word (ο ∷ ἱ ∷ []) "John.21.2"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.21.2"
∷ word (Ζ ∷ ε ∷ β ∷ ε ∷ δ ∷ α ∷ ί ∷ ο ∷ υ ∷ []) "John.21.2"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.21.2"
∷ word (ἄ ∷ ∙λ ∷ ∙λ ∷ ο ∷ ι ∷ []) "John.21.2"
∷ word (ἐ ∷ κ ∷ []) "John.21.2"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.21.2"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ ῶ ∷ ν ∷ []) "John.21.2"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.21.2"
∷ word (δ ∷ ύ ∷ ο ∷ []) "John.21.2"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.21.3"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.21.3"
∷ word (Σ ∷ ί ∷ μ ∷ ω ∷ ν ∷ []) "John.21.3"
∷ word (Π ∷ έ ∷ τ ∷ ρ ∷ ο ∷ ς ∷ []) "John.21.3"
∷ word (Ὑ ∷ π ∷ ά ∷ γ ∷ ω ∷ []) "John.21.3"
∷ word (ἁ ∷ ∙λ ∷ ι ∷ ε ∷ ύ ∷ ε ∷ ι ∷ ν ∷ []) "John.21.3"
∷ word (∙λ ∷ έ ∷ γ ∷ ο ∷ υ ∷ σ ∷ ι ∷ ν ∷ []) "John.21.3"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.21.3"
∷ word (Ἐ ∷ ρ ∷ χ ∷ ό ∷ μ ∷ ε ∷ θ ∷ α ∷ []) "John.21.3"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.21.3"
∷ word (ἡ ∷ μ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.21.3"
∷ word (σ ∷ ὺ ∷ ν ∷ []) "John.21.3"
∷ word (σ ∷ ο ∷ ί ∷ []) "John.21.3"
∷ word (ἐ ∷ ξ ∷ ῆ ∷ ∙λ ∷ θ ∷ ο ∷ ν ∷ []) "John.21.3"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.21.3"
∷ word (ἐ ∷ ν ∷ έ ∷ β ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.21.3"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.21.3"
∷ word (τ ∷ ὸ ∷ []) "John.21.3"
∷ word (π ∷ ∙λ ∷ ο ∷ ῖ ∷ ο ∷ ν ∷ []) "John.21.3"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.21.3"
∷ word (ἐ ∷ ν ∷ []) "John.21.3"
∷ word (ἐ ∷ κ ∷ ε ∷ ί ∷ ν ∷ ῃ ∷ []) "John.21.3"
∷ word (τ ∷ ῇ ∷ []) "John.21.3"
∷ word (ν ∷ υ ∷ κ ∷ τ ∷ ὶ ∷ []) "John.21.3"
∷ word (ἐ ∷ π ∷ ί ∷ α ∷ σ ∷ α ∷ ν ∷ []) "John.21.3"
∷ word (ο ∷ ὐ ∷ δ ∷ έ ∷ ν ∷ []) "John.21.3"
∷ word (Π ∷ ρ ∷ ω ∷ ΐ ∷ α ∷ ς ∷ []) "John.21.4"
∷ word (δ ∷ ὲ ∷ []) "John.21.4"
∷ word (ἤ ∷ δ ∷ η ∷ []) "John.21.4"
∷ word (γ ∷ ε ∷ ν ∷ ο ∷ μ ∷ έ ∷ ν ∷ η ∷ ς ∷ []) "John.21.4"
∷ word (ἔ ∷ σ ∷ τ ∷ η ∷ []) "John.21.4"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.21.4"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.21.4"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.21.4"
∷ word (α ∷ ἰ ∷ γ ∷ ι ∷ α ∷ ∙λ ∷ ό ∷ ν ∷ []) "John.21.4"
∷ word (ο ∷ ὐ ∷ []) "John.21.4"
∷ word (μ ∷ έ ∷ ν ∷ τ ∷ ο ∷ ι ∷ []) "John.21.4"
∷ word (ᾔ ∷ δ ∷ ε ∷ ι ∷ σ ∷ α ∷ ν ∷ []) "John.21.4"
∷ word (ο ∷ ἱ ∷ []) "John.21.4"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ α ∷ ὶ ∷ []) "John.21.4"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.21.4"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.21.4"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.21.4"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.21.5"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.21.5"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.21.5"
∷ word (ὁ ∷ []) "John.21.5"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.21.5"
∷ word (Π ∷ α ∷ ι ∷ δ ∷ ί ∷ α ∷ []) "John.21.5"
∷ word (μ ∷ ή ∷ []) "John.21.5"
∷ word (τ ∷ ι ∷ []) "John.21.5"
∷ word (π ∷ ρ ∷ ο ∷ σ ∷ φ ∷ ά ∷ γ ∷ ι ∷ ο ∷ ν ∷ []) "John.21.5"
∷ word (ἔ ∷ χ ∷ ε ∷ τ ∷ ε ∷ []) "John.21.5"
∷ word (ἀ ∷ π ∷ ε ∷ κ ∷ ρ ∷ ί ∷ θ ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.21.5"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.21.5"
∷ word (Ο ∷ ὔ ∷ []) "John.21.5"
∷ word (ὁ ∷ []) "John.21.6"
∷ word (δ ∷ ὲ ∷ []) "John.21.6"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.21.6"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.21.6"
∷ word (Β ∷ ά ∷ ∙λ ∷ ε ∷ τ ∷ ε ∷ []) "John.21.6"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.21.6"
∷ word (τ ∷ ὰ ∷ []) "John.21.6"
∷ word (δ ∷ ε ∷ ξ ∷ ι ∷ ὰ ∷ []) "John.21.6"
∷ word (μ ∷ έ ∷ ρ ∷ η ∷ []) "John.21.6"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.21.6"
∷ word (π ∷ ∙λ ∷ ο ∷ ί ∷ ο ∷ υ ∷ []) "John.21.6"
∷ word (τ ∷ ὸ ∷ []) "John.21.6"
∷ word (δ ∷ ί ∷ κ ∷ τ ∷ υ ∷ ο ∷ ν ∷ []) "John.21.6"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.21.6"
∷ word (ε ∷ ὑ ∷ ρ ∷ ή ∷ σ ∷ ε ∷ τ ∷ ε ∷ []) "John.21.6"
∷ word (ἔ ∷ β ∷ α ∷ ∙λ ∷ ο ∷ ν ∷ []) "John.21.6"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.21.6"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.21.6"
∷ word (ο ∷ ὐ ∷ κ ∷ έ ∷ τ ∷ ι ∷ []) "John.21.6"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ []) "John.21.6"
∷ word (ἑ ∷ ∙λ ∷ κ ∷ ύ ∷ σ ∷ α ∷ ι ∷ []) "John.21.6"
∷ word (ἴ ∷ σ ∷ χ ∷ υ ∷ ο ∷ ν ∷ []) "John.21.6"
∷ word (ἀ ∷ π ∷ ὸ ∷ []) "John.21.6"
∷ word (τ ∷ ο ∷ ῦ ∷ []) "John.21.6"
∷ word (π ∷ ∙λ ∷ ή ∷ θ ∷ ο ∷ υ ∷ ς ∷ []) "John.21.6"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.21.6"
∷ word (ἰ ∷ χ ∷ θ ∷ ύ ∷ ω ∷ ν ∷ []) "John.21.6"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.21.7"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.21.7"
∷ word (ὁ ∷ []) "John.21.7"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ ὴ ∷ ς ∷ []) "John.21.7"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ο ∷ ς ∷ []) "John.21.7"
∷ word (ὃ ∷ ν ∷ []) "John.21.7"
∷ word (ἠ ∷ γ ∷ ά ∷ π ∷ α ∷ []) "John.21.7"
∷ word (ὁ ∷ []) "John.21.7"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.21.7"
∷ word (τ ∷ ῷ ∷ []) "John.21.7"
∷ word (Π ∷ έ ∷ τ ∷ ρ ∷ ῳ ∷ []) "John.21.7"
∷ word (Ὁ ∷ []) "John.21.7"
∷ word (κ ∷ ύ ∷ ρ ∷ ι ∷ ό ∷ ς ∷ []) "John.21.7"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.21.7"
∷ word (Σ ∷ ί ∷ μ ∷ ω ∷ ν ∷ []) "John.21.7"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.21.7"
∷ word (Π ∷ έ ∷ τ ∷ ρ ∷ ο ∷ ς ∷ []) "John.21.7"
∷ word (ἀ ∷ κ ∷ ο ∷ ύ ∷ σ ∷ α ∷ ς ∷ []) "John.21.7"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.21.7"
∷ word (ὁ ∷ []) "John.21.7"
∷ word (κ ∷ ύ ∷ ρ ∷ ι ∷ ό ∷ ς ∷ []) "John.21.7"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.21.7"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.21.7"
∷ word (ἐ ∷ π ∷ ε ∷ ν ∷ δ ∷ ύ ∷ τ ∷ η ∷ ν ∷ []) "John.21.7"
∷ word (δ ∷ ι ∷ ε ∷ ζ ∷ ώ ∷ σ ∷ α ∷ τ ∷ ο ∷ []) "John.21.7"
∷ word (ἦ ∷ ν ∷ []) "John.21.7"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.21.7"
∷ word (γ ∷ υ ∷ μ ∷ ν ∷ ό ∷ ς ∷ []) "John.21.7"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.21.7"
∷ word (ἔ ∷ β ∷ α ∷ ∙λ ∷ ε ∷ ν ∷ []) "John.21.7"
∷ word (ἑ ∷ α ∷ υ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.21.7"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.21.7"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.21.7"
∷ word (θ ∷ ά ∷ ∙λ ∷ α ∷ σ ∷ σ ∷ α ∷ ν ∷ []) "John.21.7"
∷ word (ο ∷ ἱ ∷ []) "John.21.8"
∷ word (δ ∷ ὲ ∷ []) "John.21.8"
∷ word (ἄ ∷ ∙λ ∷ ∙λ ∷ ο ∷ ι ∷ []) "John.21.8"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ α ∷ ὶ ∷ []) "John.21.8"
∷ word (τ ∷ ῷ ∷ []) "John.21.8"
∷ word (π ∷ ∙λ ∷ ο ∷ ι ∷ α ∷ ρ ∷ ί ∷ ῳ ∷ []) "John.21.8"
∷ word (ἦ ∷ ∙λ ∷ θ ∷ ο ∷ ν ∷ []) "John.21.8"
∷ word (ο ∷ ὐ ∷ []) "John.21.8"
∷ word (γ ∷ ὰ ∷ ρ ∷ []) "John.21.8"
∷ word (ἦ ∷ σ ∷ α ∷ ν ∷ []) "John.21.8"
∷ word (μ ∷ α ∷ κ ∷ ρ ∷ ὰ ∷ ν ∷ []) "John.21.8"
∷ word (ἀ ∷ π ∷ ὸ ∷ []) "John.21.8"
∷ word (τ ∷ ῆ ∷ ς ∷ []) "John.21.8"
∷ word (γ ∷ ῆ ∷ ς ∷ []) "John.21.8"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.21.8"
∷ word (ὡ ∷ ς ∷ []) "John.21.8"
∷ word (ἀ ∷ π ∷ ὸ ∷ []) "John.21.8"
∷ word (π ∷ η ∷ χ ∷ ῶ ∷ ν ∷ []) "John.21.8"
∷ word (δ ∷ ι ∷ α ∷ κ ∷ ο ∷ σ ∷ ί ∷ ω ∷ ν ∷ []) "John.21.8"
∷ word (σ ∷ ύ ∷ ρ ∷ ο ∷ ν ∷ τ ∷ ε ∷ ς ∷ []) "John.21.8"
∷ word (τ ∷ ὸ ∷ []) "John.21.8"
∷ word (δ ∷ ί ∷ κ ∷ τ ∷ υ ∷ ο ∷ ν ∷ []) "John.21.8"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.21.8"
∷ word (ἰ ∷ χ ∷ θ ∷ ύ ∷ ω ∷ ν ∷ []) "John.21.8"
∷ word (Ὡ ∷ ς ∷ []) "John.21.9"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.21.9"
∷ word (ἀ ∷ π ∷ έ ∷ β ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.21.9"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.21.9"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.21.9"
∷ word (γ ∷ ῆ ∷ ν ∷ []) "John.21.9"
∷ word (β ∷ ∙λ ∷ έ ∷ π ∷ ο ∷ υ ∷ σ ∷ ι ∷ ν ∷ []) "John.21.9"
∷ word (ἀ ∷ ν ∷ θ ∷ ρ ∷ α ∷ κ ∷ ι ∷ ὰ ∷ ν ∷ []) "John.21.9"
∷ word (κ ∷ ε ∷ ι ∷ μ ∷ έ ∷ ν ∷ η ∷ ν ∷ []) "John.21.9"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.21.9"
∷ word (ὀ ∷ ψ ∷ ά ∷ ρ ∷ ι ∷ ο ∷ ν ∷ []) "John.21.9"
∷ word (ἐ ∷ π ∷ ι ∷ κ ∷ ε ∷ ί ∷ μ ∷ ε ∷ ν ∷ ο ∷ ν ∷ []) "John.21.9"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.21.9"
∷ word (ἄ ∷ ρ ∷ τ ∷ ο ∷ ν ∷ []) "John.21.9"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.21.10"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.21.10"
∷ word (ὁ ∷ []) "John.21.10"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.21.10"
∷ word (Ἐ ∷ ν ∷ έ ∷ γ ∷ κ ∷ α ∷ τ ∷ ε ∷ []) "John.21.10"
∷ word (ἀ ∷ π ∷ ὸ ∷ []) "John.21.10"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.21.10"
∷ word (ὀ ∷ ψ ∷ α ∷ ρ ∷ ί ∷ ω ∷ ν ∷ []) "John.21.10"
∷ word (ὧ ∷ ν ∷ []) "John.21.10"
∷ word (ἐ ∷ π ∷ ι ∷ ά ∷ σ ∷ α ∷ τ ∷ ε ∷ []) "John.21.10"
∷ word (ν ∷ ῦ ∷ ν ∷ []) "John.21.10"
∷ word (ἀ ∷ ν ∷ έ ∷ β ∷ η ∷ []) "John.21.11"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.21.11"
∷ word (Σ ∷ ί ∷ μ ∷ ω ∷ ν ∷ []) "John.21.11"
∷ word (Π ∷ έ ∷ τ ∷ ρ ∷ ο ∷ ς ∷ []) "John.21.11"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.21.11"
∷ word (ε ∷ ἵ ∷ ∙λ ∷ κ ∷ υ ∷ σ ∷ ε ∷ ν ∷ []) "John.21.11"
∷ word (τ ∷ ὸ ∷ []) "John.21.11"
∷ word (δ ∷ ί ∷ κ ∷ τ ∷ υ ∷ ο ∷ ν ∷ []) "John.21.11"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.21.11"
∷ word (τ ∷ ὴ ∷ ν ∷ []) "John.21.11"
∷ word (γ ∷ ῆ ∷ ν ∷ []) "John.21.11"
∷ word (μ ∷ ε ∷ σ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.21.11"
∷ word (ἰ ∷ χ ∷ θ ∷ ύ ∷ ω ∷ ν ∷ []) "John.21.11"
∷ word (μ ∷ ε ∷ γ ∷ ά ∷ ∙λ ∷ ω ∷ ν ∷ []) "John.21.11"
∷ word (ἑ ∷ κ ∷ α ∷ τ ∷ ὸ ∷ ν ∷ []) "John.21.11"
∷ word (π ∷ ε ∷ ν ∷ τ ∷ ή ∷ κ ∷ ο ∷ ν ∷ τ ∷ α ∷ []) "John.21.11"
∷ word (τ ∷ ρ ∷ ι ∷ ῶ ∷ ν ∷ []) "John.21.11"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.21.11"
∷ word (τ ∷ ο ∷ σ ∷ ο ∷ ύ ∷ τ ∷ ω ∷ ν ∷ []) "John.21.11"
∷ word (ὄ ∷ ν ∷ τ ∷ ω ∷ ν ∷ []) "John.21.11"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.21.11"
∷ word (ἐ ∷ σ ∷ χ ∷ ί ∷ σ ∷ θ ∷ η ∷ []) "John.21.11"
∷ word (τ ∷ ὸ ∷ []) "John.21.11"
∷ word (δ ∷ ί ∷ κ ∷ τ ∷ υ ∷ ο ∷ ν ∷ []) "John.21.11"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.21.12"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.21.12"
∷ word (ὁ ∷ []) "John.21.12"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.21.12"
∷ word (Δ ∷ ε ∷ ῦ ∷ τ ∷ ε ∷ []) "John.21.12"
∷ word (ἀ ∷ ρ ∷ ι ∷ σ ∷ τ ∷ ή ∷ σ ∷ α ∷ τ ∷ ε ∷ []) "John.21.12"
∷ word (ο ∷ ὐ ∷ δ ∷ ε ∷ ὶ ∷ ς ∷ []) "John.21.12"
∷ word (δ ∷ ὲ ∷ []) "John.21.12"
∷ word (ἐ ∷ τ ∷ ό ∷ ∙λ ∷ μ ∷ α ∷ []) "John.21.12"
∷ word (τ ∷ ῶ ∷ ν ∷ []) "John.21.12"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ ῶ ∷ ν ∷ []) "John.21.12"
∷ word (ἐ ∷ ξ ∷ ε ∷ τ ∷ ά ∷ σ ∷ α ∷ ι ∷ []) "John.21.12"
∷ word (α ∷ ὐ ∷ τ ∷ ό ∷ ν ∷ []) "John.21.12"
∷ word (Σ ∷ ὺ ∷ []) "John.21.12"
∷ word (τ ∷ ί ∷ ς ∷ []) "John.21.12"
∷ word (ε ∷ ἶ ∷ []) "John.21.12"
∷ word (ε ∷ ἰ ∷ δ ∷ ό ∷ τ ∷ ε ∷ ς ∷ []) "John.21.12"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.21.12"
∷ word (ὁ ∷ []) "John.21.12"
∷ word (κ ∷ ύ ∷ ρ ∷ ι ∷ ό ∷ ς ∷ []) "John.21.12"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.21.12"
∷ word (ἔ ∷ ρ ∷ χ ∷ ε ∷ τ ∷ α ∷ ι ∷ []) "John.21.13"
∷ word (ὁ ∷ []) "John.21.13"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.21.13"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.21.13"
∷ word (∙λ ∷ α ∷ μ ∷ β ∷ ά ∷ ν ∷ ε ∷ ι ∷ []) "John.21.13"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.21.13"
∷ word (ἄ ∷ ρ ∷ τ ∷ ο ∷ ν ∷ []) "John.21.13"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.21.13"
∷ word (δ ∷ ί ∷ δ ∷ ω ∷ σ ∷ ι ∷ ν ∷ []) "John.21.13"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.21.13"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.21.13"
∷ word (τ ∷ ὸ ∷ []) "John.21.13"
∷ word (ὀ ∷ ψ ∷ ά ∷ ρ ∷ ι ∷ ο ∷ ν ∷ []) "John.21.13"
∷ word (ὁ ∷ μ ∷ ο ∷ ί ∷ ω ∷ ς ∷ []) "John.21.13"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.21.14"
∷ word (ἤ ∷ δ ∷ η ∷ []) "John.21.14"
∷ word (τ ∷ ρ ∷ ί ∷ τ ∷ ο ∷ ν ∷ []) "John.21.14"
∷ word (ἐ ∷ φ ∷ α ∷ ν ∷ ε ∷ ρ ∷ ώ ∷ θ ∷ η ∷ []) "John.21.14"
∷ word (ὁ ∷ []) "John.21.14"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.21.14"
∷ word (τ ∷ ο ∷ ῖ ∷ ς ∷ []) "John.21.14"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ α ∷ ῖ ∷ ς ∷ []) "John.21.14"
∷ word (ἐ ∷ γ ∷ ε ∷ ρ ∷ θ ∷ ε ∷ ὶ ∷ ς ∷ []) "John.21.14"
∷ word (ἐ ∷ κ ∷ []) "John.21.14"
∷ word (ν ∷ ε ∷ κ ∷ ρ ∷ ῶ ∷ ν ∷ []) "John.21.14"
∷ word (Ὅ ∷ τ ∷ ε ∷ []) "John.21.15"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.21.15"
∷ word (ἠ ∷ ρ ∷ ί ∷ σ ∷ τ ∷ η ∷ σ ∷ α ∷ ν ∷ []) "John.21.15"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.21.15"
∷ word (τ ∷ ῷ ∷ []) "John.21.15"
∷ word (Σ ∷ ί ∷ μ ∷ ω ∷ ν ∷ ι ∷ []) "John.21.15"
∷ word (Π ∷ έ ∷ τ ∷ ρ ∷ ῳ ∷ []) "John.21.15"
∷ word (ὁ ∷ []) "John.21.15"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.21.15"
∷ word (Σ ∷ ί ∷ μ ∷ ω ∷ ν ∷ []) "John.21.15"
∷ word (Ἰ ∷ ω ∷ ά ∷ ν ∷ ν ∷ ο ∷ υ ∷ []) "John.21.15"
∷ word (ἀ ∷ γ ∷ α ∷ π ∷ ᾷ ∷ ς ∷ []) "John.21.15"
∷ word (μ ∷ ε ∷ []) "John.21.15"
∷ word (π ∷ ∙λ ∷ έ ∷ ο ∷ ν ∷ []) "John.21.15"
∷ word (τ ∷ ο ∷ ύ ∷ τ ∷ ω ∷ ν ∷ []) "John.21.15"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.21.15"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.21.15"
∷ word (Ν ∷ α ∷ ί ∷ []) "John.21.15"
∷ word (κ ∷ ύ ∷ ρ ∷ ι ∷ ε ∷ []) "John.21.15"
∷ word (σ ∷ ὺ ∷ []) "John.21.15"
∷ word (ο ∷ ἶ ∷ δ ∷ α ∷ ς ∷ []) "John.21.15"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.21.15"
∷ word (φ ∷ ι ∷ ∙λ ∷ ῶ ∷ []) "John.21.15"
∷ word (σ ∷ ε ∷ []) "John.21.15"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.21.15"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.21.15"
∷ word (Β ∷ ό ∷ σ ∷ κ ∷ ε ∷ []) "John.21.15"
∷ word (τ ∷ ὰ ∷ []) "John.21.15"
∷ word (ἀ ∷ ρ ∷ ν ∷ ί ∷ α ∷ []) "John.21.15"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.21.15"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.21.16"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.21.16"
∷ word (π ∷ ά ∷ ∙λ ∷ ι ∷ ν ∷ []) "John.21.16"
∷ word (δ ∷ ε ∷ ύ ∷ τ ∷ ε ∷ ρ ∷ ο ∷ ν ∷ []) "John.21.16"
∷ word (Σ ∷ ί ∷ μ ∷ ω ∷ ν ∷ []) "John.21.16"
∷ word (Ἰ ∷ ω ∷ ά ∷ ν ∷ ν ∷ ο ∷ υ ∷ []) "John.21.16"
∷ word (ἀ ∷ γ ∷ α ∷ π ∷ ᾷ ∷ ς ∷ []) "John.21.16"
∷ word (μ ∷ ε ∷ []) "John.21.16"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.21.16"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.21.16"
∷ word (Ν ∷ α ∷ ί ∷ []) "John.21.16"
∷ word (κ ∷ ύ ∷ ρ ∷ ι ∷ ε ∷ []) "John.21.16"
∷ word (σ ∷ ὺ ∷ []) "John.21.16"
∷ word (ο ∷ ἶ ∷ δ ∷ α ∷ ς ∷ []) "John.21.16"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.21.16"
∷ word (φ ∷ ι ∷ ∙λ ∷ ῶ ∷ []) "John.21.16"
∷ word (σ ∷ ε ∷ []) "John.21.16"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.21.16"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.21.16"
∷ word (Π ∷ ο ∷ ί ∷ μ ∷ α ∷ ι ∷ ν ∷ ε ∷ []) "John.21.16"
∷ word (τ ∷ ὰ ∷ []) "John.21.16"
∷ word (π ∷ ρ ∷ ό ∷ β ∷ α ∷ τ ∷ ά ∷ []) "John.21.16"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.21.16"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.21.17"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.21.17"
∷ word (τ ∷ ὸ ∷ []) "John.21.17"
∷ word (τ ∷ ρ ∷ ί ∷ τ ∷ ο ∷ ν ∷ []) "John.21.17"
∷ word (Σ ∷ ί ∷ μ ∷ ω ∷ ν ∷ []) "John.21.17"
∷ word (Ἰ ∷ ω ∷ ά ∷ ν ∷ ν ∷ ο ∷ υ ∷ []) "John.21.17"
∷ word (φ ∷ ι ∷ ∙λ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.21.17"
∷ word (μ ∷ ε ∷ []) "John.21.17"
∷ word (ἐ ∷ ∙λ ∷ υ ∷ π ∷ ή ∷ θ ∷ η ∷ []) "John.21.17"
∷ word (ὁ ∷ []) "John.21.17"
∷ word (Π ∷ έ ∷ τ ∷ ρ ∷ ο ∷ ς ∷ []) "John.21.17"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.21.17"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.21.17"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.21.17"
∷ word (τ ∷ ὸ ∷ []) "John.21.17"
∷ word (τ ∷ ρ ∷ ί ∷ τ ∷ ο ∷ ν ∷ []) "John.21.17"
∷ word (Φ ∷ ι ∷ ∙λ ∷ ε ∷ ῖ ∷ ς ∷ []) "John.21.17"
∷ word (μ ∷ ε ∷ []) "John.21.17"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.21.17"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.21.17"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.21.17"
∷ word (Κ ∷ ύ ∷ ρ ∷ ι ∷ ε ∷ []) "John.21.17"
∷ word (π ∷ ά ∷ ν ∷ τ ∷ α ∷ []) "John.21.17"
∷ word (σ ∷ ὺ ∷ []) "John.21.17"
∷ word (ο ∷ ἶ ∷ δ ∷ α ∷ ς ∷ []) "John.21.17"
∷ word (σ ∷ ὺ ∷ []) "John.21.17"
∷ word (γ ∷ ι ∷ ν ∷ ώ ∷ σ ∷ κ ∷ ε ∷ ι ∷ ς ∷ []) "John.21.17"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.21.17"
∷ word (φ ∷ ι ∷ ∙λ ∷ ῶ ∷ []) "John.21.17"
∷ word (σ ∷ ε ∷ []) "John.21.17"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.21.17"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.21.17"
∷ word (ὁ ∷ []) "John.21.17"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.21.17"
∷ word (Β ∷ ό ∷ σ ∷ κ ∷ ε ∷ []) "John.21.17"
∷ word (τ ∷ ὰ ∷ []) "John.21.17"
∷ word (π ∷ ρ ∷ ό ∷ β ∷ α ∷ τ ∷ ά ∷ []) "John.21.17"
∷ word (μ ∷ ο ∷ υ ∷ []) "John.21.17"
∷ word (ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.21.18"
∷ word (ἀ ∷ μ ∷ ὴ ∷ ν ∷ []) "John.21.18"
∷ word (∙λ ∷ έ ∷ γ ∷ ω ∷ []) "John.21.18"
∷ word (σ ∷ ο ∷ ι ∷ []) "John.21.18"
∷ word (ὅ ∷ τ ∷ ε ∷ []) "John.21.18"
∷ word (ἦ ∷ ς ∷ []) "John.21.18"
∷ word (ν ∷ ε ∷ ώ ∷ τ ∷ ε ∷ ρ ∷ ο ∷ ς ∷ []) "John.21.18"
∷ word (ἐ ∷ ζ ∷ ώ ∷ ν ∷ ν ∷ υ ∷ ε ∷ ς ∷ []) "John.21.18"
∷ word (σ ∷ ε ∷ α ∷ υ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.21.18"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.21.18"
∷ word (π ∷ ε ∷ ρ ∷ ι ∷ ε ∷ π ∷ ά ∷ τ ∷ ε ∷ ι ∷ ς ∷ []) "John.21.18"
∷ word (ὅ ∷ π ∷ ο ∷ υ ∷ []) "John.21.18"
∷ word (ἤ ∷ θ ∷ ε ∷ ∙λ ∷ ε ∷ ς ∷ []) "John.21.18"
∷ word (ὅ ∷ τ ∷ α ∷ ν ∷ []) "John.21.18"
∷ word (δ ∷ ὲ ∷ []) "John.21.18"
∷ word (γ ∷ η ∷ ρ ∷ ά ∷ σ ∷ ῃ ∷ ς ∷ []) "John.21.18"
∷ word (ἐ ∷ κ ∷ τ ∷ ε ∷ ν ∷ ε ∷ ῖ ∷ ς ∷ []) "John.21.18"
∷ word (τ ∷ ὰ ∷ ς ∷ []) "John.21.18"
∷ word (χ ∷ ε ∷ ῖ ∷ ρ ∷ ά ∷ ς ∷ []) "John.21.18"
∷ word (σ ∷ ο ∷ υ ∷ []) "John.21.18"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.21.18"
∷ word (ἄ ∷ ∙λ ∷ ∙λ ∷ ο ∷ ς ∷ []) "John.21.18"
∷ word (σ ∷ ε ∷ []) "John.21.18"
∷ word (ζ ∷ ώ ∷ σ ∷ ε ∷ ι ∷ []) "John.21.18"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.21.18"
∷ word (ο ∷ ἴ ∷ σ ∷ ε ∷ ι ∷ []) "John.21.18"
∷ word (ὅ ∷ π ∷ ο ∷ υ ∷ []) "John.21.18"
∷ word (ο ∷ ὐ ∷ []) "John.21.18"
∷ word (θ ∷ έ ∷ ∙λ ∷ ε ∷ ι ∷ ς ∷ []) "John.21.18"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.21.19"
∷ word (δ ∷ ὲ ∷ []) "John.21.19"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.21.19"
∷ word (σ ∷ η ∷ μ ∷ α ∷ ί ∷ ν ∷ ω ∷ ν ∷ []) "John.21.19"
∷ word (π ∷ ο ∷ ί ∷ ῳ ∷ []) "John.21.19"
∷ word (θ ∷ α ∷ ν ∷ ά ∷ τ ∷ ῳ ∷ []) "John.21.19"
∷ word (δ ∷ ο ∷ ξ ∷ ά ∷ σ ∷ ε ∷ ι ∷ []) "John.21.19"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.21.19"
∷ word (θ ∷ ε ∷ ό ∷ ν ∷ []) "John.21.19"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.21.19"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ []) "John.21.19"
∷ word (ε ∷ ἰ ∷ π ∷ ὼ ∷ ν ∷ []) "John.21.19"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.21.19"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.21.19"
∷ word (Ἀ ∷ κ ∷ ο ∷ ∙λ ∷ ο ∷ ύ ∷ θ ∷ ε ∷ ι ∷ []) "John.21.19"
∷ word (μ ∷ ο ∷ ι ∷ []) "John.21.19"
∷ word (Ἐ ∷ π ∷ ι ∷ σ ∷ τ ∷ ρ ∷ α ∷ φ ∷ ε ∷ ὶ ∷ ς ∷ []) "John.21.20"
∷ word (ὁ ∷ []) "John.21.20"
∷ word (Π ∷ έ ∷ τ ∷ ρ ∷ ο ∷ ς ∷ []) "John.21.20"
∷ word (β ∷ ∙λ ∷ έ ∷ π ∷ ε ∷ ι ∷ []) "John.21.20"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.21.20"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ ὴ ∷ ν ∷ []) "John.21.20"
∷ word (ὃ ∷ ν ∷ []) "John.21.20"
∷ word (ἠ ∷ γ ∷ ά ∷ π ∷ α ∷ []) "John.21.20"
∷ word (ὁ ∷ []) "John.21.20"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.21.20"
∷ word (ἀ ∷ κ ∷ ο ∷ ∙λ ∷ ο ∷ υ ∷ θ ∷ ο ∷ ῦ ∷ ν ∷ τ ∷ α ∷ []) "John.21.20"
∷ word (ὃ ∷ ς ∷ []) "John.21.20"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.21.20"
∷ word (ἀ ∷ ν ∷ έ ∷ π ∷ ε ∷ σ ∷ ε ∷ ν ∷ []) "John.21.20"
∷ word (ἐ ∷ ν ∷ []) "John.21.20"
∷ word (τ ∷ ῷ ∷ []) "John.21.20"
∷ word (δ ∷ ε ∷ ί ∷ π ∷ ν ∷ ῳ ∷ []) "John.21.20"
∷ word (ἐ ∷ π ∷ ὶ ∷ []) "John.21.20"
∷ word (τ ∷ ὸ ∷ []) "John.21.20"
∷ word (σ ∷ τ ∷ ῆ ∷ θ ∷ ο ∷ ς ∷ []) "John.21.20"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.21.20"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.21.20"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.21.20"
∷ word (Κ ∷ ύ ∷ ρ ∷ ι ∷ ε ∷ []) "John.21.20"
∷ word (τ ∷ ί ∷ ς ∷ []) "John.21.20"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.21.20"
∷ word (ὁ ∷ []) "John.21.20"
∷ word (π ∷ α ∷ ρ ∷ α ∷ δ ∷ ι ∷ δ ∷ ο ∷ ύ ∷ ς ∷ []) "John.21.20"
∷ word (σ ∷ ε ∷ []) "John.21.20"
∷ word (τ ∷ ο ∷ ῦ ∷ τ ∷ ο ∷ ν ∷ []) "John.21.21"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.21.21"
∷ word (ἰ ∷ δ ∷ ὼ ∷ ν ∷ []) "John.21.21"
∷ word (ὁ ∷ []) "John.21.21"
∷ word (Π ∷ έ ∷ τ ∷ ρ ∷ ο ∷ ς ∷ []) "John.21.21"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.21.21"
∷ word (τ ∷ ῷ ∷ []) "John.21.21"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ []) "John.21.21"
∷ word (Κ ∷ ύ ∷ ρ ∷ ι ∷ ε ∷ []) "John.21.21"
∷ word (ο ∷ ὗ ∷ τ ∷ ο ∷ ς ∷ []) "John.21.21"
∷ word (δ ∷ ὲ ∷ []) "John.21.21"
∷ word (τ ∷ ί ∷ []) "John.21.21"
∷ word (∙λ ∷ έ ∷ γ ∷ ε ∷ ι ∷ []) "John.21.22"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.21.22"
∷ word (ὁ ∷ []) "John.21.22"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.21.22"
∷ word (Ἐ ∷ ὰ ∷ ν ∷ []) "John.21.22"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.21.22"
∷ word (θ ∷ έ ∷ ∙λ ∷ ω ∷ []) "John.21.22"
∷ word (μ ∷ έ ∷ ν ∷ ε ∷ ι ∷ ν ∷ []) "John.21.22"
∷ word (ἕ ∷ ω ∷ ς ∷ []) "John.21.22"
∷ word (ἔ ∷ ρ ∷ χ ∷ ο ∷ μ ∷ α ∷ ι ∷ []) "John.21.22"
∷ word (τ ∷ ί ∷ []) "John.21.22"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.21.22"
∷ word (σ ∷ έ ∷ []) "John.21.22"
∷ word (σ ∷ ύ ∷ []) "John.21.22"
∷ word (μ ∷ ο ∷ ι ∷ []) "John.21.22"
∷ word (ἀ ∷ κ ∷ ο ∷ ∙λ ∷ ο ∷ ύ ∷ θ ∷ ε ∷ ι ∷ []) "John.21.22"
∷ word (ἐ ∷ ξ ∷ ῆ ∷ ∙λ ∷ θ ∷ ε ∷ ν ∷ []) "John.21.23"
∷ word (ο ∷ ὖ ∷ ν ∷ []) "John.21.23"
∷ word (ο ∷ ὗ ∷ τ ∷ ο ∷ ς ∷ []) "John.21.23"
∷ word (ὁ ∷ []) "John.21.23"
∷ word (∙λ ∷ ό ∷ γ ∷ ο ∷ ς ∷ []) "John.21.23"
∷ word (ε ∷ ἰ ∷ ς ∷ []) "John.21.23"
∷ word (τ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.21.23"
∷ word (ἀ ∷ δ ∷ ε ∷ ∙λ ∷ φ ∷ ο ∷ ὺ ∷ ς ∷ []) "John.21.23"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.21.23"
∷ word (ὁ ∷ []) "John.21.23"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ ὴ ∷ ς ∷ []) "John.21.23"
∷ word (ἐ ∷ κ ∷ ε ∷ ῖ ∷ ν ∷ ο ∷ ς ∷ []) "John.21.23"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.21.23"
∷ word (ἀ ∷ π ∷ ο ∷ θ ∷ ν ∷ ῄ ∷ σ ∷ κ ∷ ε ∷ ι ∷ []) "John.21.23"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.21.23"
∷ word (ε ∷ ἶ ∷ π ∷ ε ∷ ν ∷ []) "John.21.23"
∷ word (δ ∷ ὲ ∷ []) "John.21.23"
∷ word (α ∷ ὐ ∷ τ ∷ ῷ ∷ []) "John.21.23"
∷ word (ὁ ∷ []) "John.21.23"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.21.23"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.21.23"
∷ word (ο ∷ ὐ ∷ κ ∷ []) "John.21.23"
∷ word (ἀ ∷ π ∷ ο ∷ θ ∷ ν ∷ ῄ ∷ σ ∷ κ ∷ ε ∷ ι ∷ []) "John.21.23"
∷ word (ἀ ∷ ∙λ ∷ ∙λ ∷ []) "John.21.23"
∷ word (Ἐ ∷ ὰ ∷ ν ∷ []) "John.21.23"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.21.23"
∷ word (θ ∷ έ ∷ ∙λ ∷ ω ∷ []) "John.21.23"
∷ word (μ ∷ έ ∷ ν ∷ ε ∷ ι ∷ ν ∷ []) "John.21.23"
∷ word (ἕ ∷ ω ∷ ς ∷ []) "John.21.23"
∷ word (ἔ ∷ ρ ∷ χ ∷ ο ∷ μ ∷ α ∷ ι ∷ []) "John.21.23"
∷ word (τ ∷ ί ∷ []) "John.21.23"
∷ word (π ∷ ρ ∷ ὸ ∷ ς ∷ []) "John.21.23"
∷ word (σ ∷ έ ∷ []) "John.21.23"
∷ word (Ο ∷ ὗ ∷ τ ∷ ό ∷ ς ∷ []) "John.21.24"
∷ word (ἐ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.21.24"
∷ word (ὁ ∷ []) "John.21.24"
∷ word (μ ∷ α ∷ θ ∷ η ∷ τ ∷ ὴ ∷ ς ∷ []) "John.21.24"
∷ word (ὁ ∷ []) "John.21.24"
∷ word (μ ∷ α ∷ ρ ∷ τ ∷ υ ∷ ρ ∷ ῶ ∷ ν ∷ []) "John.21.24"
∷ word (π ∷ ε ∷ ρ ∷ ὶ ∷ []) "John.21.24"
∷ word (τ ∷ ο ∷ ύ ∷ τ ∷ ω ∷ ν ∷ []) "John.21.24"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.21.24"
∷ word (ὁ ∷ []) "John.21.24"
∷ word (γ ∷ ρ ∷ ά ∷ ψ ∷ α ∷ ς ∷ []) "John.21.24"
∷ word (τ ∷ α ∷ ῦ ∷ τ ∷ α ∷ []) "John.21.24"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.21.24"
∷ word (ο ∷ ἴ ∷ δ ∷ α ∷ μ ∷ ε ∷ ν ∷ []) "John.21.24"
∷ word (ὅ ∷ τ ∷ ι ∷ []) "John.21.24"
∷ word (ἀ ∷ ∙λ ∷ η ∷ θ ∷ ὴ ∷ ς ∷ []) "John.21.24"
∷ word (α ∷ ὐ ∷ τ ∷ ο ∷ ῦ ∷ []) "John.21.24"
∷ word (ἡ ∷ []) "John.21.24"
∷ word (μ ∷ α ∷ ρ ∷ τ ∷ υ ∷ ρ ∷ ί ∷ α ∷ []) "John.21.24"
∷ word (ἐ ∷ σ ∷ τ ∷ ί ∷ ν ∷ []) "John.21.24"
∷ word (ἔ ∷ σ ∷ τ ∷ ι ∷ ν ∷ []) "John.21.25"
∷ word (δ ∷ ὲ ∷ []) "John.21.25"
∷ word (κ ∷ α ∷ ὶ ∷ []) "John.21.25"
∷ word (ἄ ∷ ∙λ ∷ ∙λ ∷ α ∷ []) "John.21.25"
∷ word (π ∷ ο ∷ ∙λ ∷ ∙λ ∷ ὰ ∷ []) "John.21.25"
∷ word (ἃ ∷ []) "John.21.25"
∷ word (ἐ ∷ π ∷ ο ∷ ί ∷ η ∷ σ ∷ ε ∷ ν ∷ []) "John.21.25"
∷ word (ὁ ∷ []) "John.21.25"
∷ word (Ἰ ∷ η ∷ σ ∷ ο ∷ ῦ ∷ ς ∷ []) "John.21.25"
∷ word (ἅ ∷ τ ∷ ι ∷ ν ∷ α ∷ []) "John.21.25"
∷ word (ἐ ∷ ὰ ∷ ν ∷ []) "John.21.25"
∷ word (γ ∷ ρ ∷ ά ∷ φ ∷ η ∷ τ ∷ α ∷ ι ∷ []) "John.21.25"
∷ word (κ ∷ α ∷ θ ∷ []) "John.21.25"
∷ word (ἕ ∷ ν ∷ []) "John.21.25"
∷ word (ο ∷ ὐ ∷ δ ∷ []) "John.21.25"
∷ word (α ∷ ὐ ∷ τ ∷ ὸ ∷ ν ∷ []) "John.21.25"
∷ word (ο ∷ ἶ ∷ μ ∷ α ∷ ι ∷ []) "John.21.25"
∷ word (τ ∷ ὸ ∷ ν ∷ []) "John.21.25"
∷ word (κ ∷ ό ∷ σ ∷ μ ∷ ο ∷ ν ∷ []) "John.21.25"
∷ word (χ ∷ ω ∷ ρ ∷ ή ∷ σ ∷ ε ∷ ι ∷ ν ∷ []) "John.21.25"
∷ word (τ ∷ ὰ ∷ []) "John.21.25"
∷ word (γ ∷ ρ ∷ α ∷ φ ∷ ό ∷ μ ∷ ε ∷ ν ∷ α ∷ []) "John.21.25"
∷ word (β ∷ ι ∷ β ∷ ∙λ ∷ ί ∷ α ∷ []) "John.21.25"
∷ []
| {
"alphanum_fraction": 0.3556474991,
"avg_line_length": 44.6811444106,
"ext": "agda",
"hexsha": "ebeb8f9f4cb0f51299ffc42f9e0827d60eb4f1b5",
"lang": "Agda",
"max_forks_count": 5,
"max_forks_repo_forks_event_max_datetime": "2017-06-11T11:25:09.000Z",
"max_forks_repo_forks_event_min_datetime": "2015-02-27T22:34:13.000Z",
"max_forks_repo_head_hexsha": "915c46c27c7f8aad5907474d8484f2685a4cd6a7",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "scott-fleischman/GreekGrammar",
"max_forks_repo_path": "agda/Text/Greek/SBLGNT/John.agda",
"max_issues_count": 13,
"max_issues_repo_head_hexsha": "915c46c27c7f8aad5907474d8484f2685a4cd6a7",
"max_issues_repo_issues_event_max_datetime": "2020-09-07T11:58:38.000Z",
"max_issues_repo_issues_event_min_datetime": "2015-05-28T20:04:08.000Z",
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "scott-fleischman/GreekGrammar",
"max_issues_repo_path": "agda/Text/Greek/SBLGNT/John.agda",
"max_line_length": 89,
"max_stars_count": 44,
"max_stars_repo_head_hexsha": "915c46c27c7f8aad5907474d8484f2685a4cd6a7",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "scott-fleischman/GreekGrammar",
"max_stars_repo_path": "agda/Text/Greek/SBLGNT/John.agda",
"max_stars_repo_stars_event_max_datetime": "2022-03-06T15:41:57.000Z",
"max_stars_repo_stars_event_min_datetime": "2015-05-29T14:48:51.000Z",
"num_tokens": 466183,
"size": 690279
} |
{-# OPTIONS --without-K #-}
open import Data.Bits.Search
open import Data.Nat.NP
open import Function.NP
import Relation.Binary.PropositionalEquality.NP as ≡
open ≡
module Data.Bits.Sum where
open SimpleSearch _+_ using (module Comm; module SearchInterchange; module SearchUnit; module Bij)
open SimpleSearch _+_ public using () renaming (search to sum; search-≗ to sum-≗; searchBit to sumBit;
search-≗₂ to sum-≗₂;
search-+ to sum-+)
open Comm ℕ°.+-comm public renaming (search-comm to sum-comm)
open SearchUnit 0 refl public renaming
(search-constε≡ε to sum-const0≡0)
open SearchInterchange +-interchange public renaming (
search-dist to sum-dist;
search-searchBit to sum-sumBit;
search-search to sum-sum;
search-swap to sum-swap)
open Bij ℕ°.+-comm +-interchange public renaming (search-bij to sum-bij)
sum-const : ∀ n x → sum {n} (const x) ≡ ⟨2^ n * x ⟩
sum-const zero _ = refl
sum-const (suc n) x = cong₂ _+_ (sum-const n x) (sum-const n x)
| {
"alphanum_fraction": 0.617152962,
"avg_line_length": 40.3928571429,
"ext": "agda",
"hexsha": "b6de0cda444644b62a8de95937e3defc77aaa895",
"lang": "Agda",
"max_forks_count": null,
"max_forks_repo_forks_event_max_datetime": null,
"max_forks_repo_forks_event_min_datetime": null,
"max_forks_repo_head_hexsha": "16bc8333503ff9c00d47d56f4ec6113b9269a43e",
"max_forks_repo_licenses": [
"BSD-3-Clause"
],
"max_forks_repo_name": "crypto-agda/explore",
"max_forks_repo_path": "lib/Explore/Experimental/DataBitsSum.agda",
"max_issues_count": 1,
"max_issues_repo_head_hexsha": "16bc8333503ff9c00d47d56f4ec6113b9269a43e",
"max_issues_repo_issues_event_max_datetime": "2019-03-16T14:24:04.000Z",
"max_issues_repo_issues_event_min_datetime": "2019-03-16T14:24:04.000Z",
"max_issues_repo_licenses": [
"BSD-3-Clause"
],
"max_issues_repo_name": "crypto-agda/explore",
"max_issues_repo_path": "lib/Explore/Experimental/DataBitsSum.agda",
"max_line_length": 106,
"max_stars_count": 2,
"max_stars_repo_head_hexsha": "16bc8333503ff9c00d47d56f4ec6113b9269a43e",
"max_stars_repo_licenses": [
"BSD-3-Clause"
],
"max_stars_repo_name": "crypto-agda/explore",
"max_stars_repo_path": "lib/Explore/Experimental/DataBitsSum.agda",
"max_stars_repo_stars_event_max_datetime": "2017-06-28T19:19:29.000Z",
"max_stars_repo_stars_event_min_datetime": "2016-06-05T09:25:32.000Z",
"num_tokens": 304,
"size": 1131
} |
module x05isomorphism where
{-
------------------------------------------------------------------------------
Isomorphism: Isomorphism and Embedding
isomorphism
- way of asserting two types are equal
embedding
- way of asserting that one type is smaller than another
apply isomorphisms in next chapter to show 'product' and 'sum' satisfy properties
similar to associativity, commutativity, and distributivity
-}
import Relation.Binary.PropositionalEquality as Eq
open Eq using (_≡_; refl; cong; cong-app)
open Eq.≡-Reasoning
open import Data.Nat using (ℕ; zero; suc; _+_)
open import Data.Nat.Properties using (+-comm)
{-
------------------------------------------------------------------------------
LAMBDA EXPRESSIONS : ANONYMOUS FUNS
λ{ P₁ → N₁; ⋯ ; Ppₙ → Np }
equivalent def by equations
f P₁ = N₁
⋯
f Pp = Npₙ
where
- P are patterns (left-hand sides of an equation)
- N are expressions (right-hand side of an equation)
for case of one equation and pattern is a variable:
λ x → N
or
λ (x : A) → N
equivalent to
λ{x → N}
------------------------------------------------------------------------------
Function composition
-}
-- first apply f, then apply g to result
_∘_ : ∀ {A B C : Set} → (B → C) → (A → B) → (A → C)
(g ∘ f) x = g (f x)
-- equivalent
_∘′_ : ∀ {A B C : Set} → (B → C) → (A → B) → (A → C)
g ∘′ f = λ x → g (f x)
{-
------------------------------------------------------------------------------
EXTENSIONALITY : only way to distinguish functions is by applying them
If two functions applied to same arg always give same result, then they are same.
converse of cong-app
Agda does not presume extensionality, so
-}
postulate
extensionality : ∀ {A B : Set} {f g : A → B}
→ (∀ (x : A) → f x ≡ g x)
-----------------------
→ f ≡ g
{-
Postulating extensionality does not lead to difficulties.
It is known to be consistent with the theory that underlies Agda.
example
-}
-- version that matches on right
_+′_ : ℕ → ℕ → ℕ
m +′ zero = m
m +′ suc n = suc (m +′ n)
-- using commutativity, show + and +′ always return same result for same arg
same-app : ∀ (m n : ℕ) → m +′ n ≡ m + n
same-app m n -- (m +′ n) ≡ m + n
rewrite +-comm m n -- (m +′ n) ≡ n + m
= helper m n
where
helper : ∀ (m n : ℕ) → m +′ n ≡ n + m
helper m zero = refl
helper m (suc n) -- suc (m +′ n) ≡ suc (n + m)
= cong suc (helper m n)
-- now assert + and +′ to be indistinguishable (via two applications of extensionality)
same : _+′_ ≡ _+_
same = extensionality (λ m → extensionality (λ n → same-app m n))
{-
to postulate extensionality in what follows
(and to postulate extensionality for dependent functions):
-}
-- type of f and g has changed from A → B to ∀ (x : A) → B x
postulate
∀-extensionality : ∀ {A : Set} {B : A → Set} {f g : ∀(x : A) → B x}
→ (∀ (x : A) → f x ≡ g x)
-----------------------
→ f ≡ g
{-
------------------------------------------------------------------------------
ISOMORPHISM : sets are isomorphic if they are in one-to-one correspondence
formal definition:
-}
infix 0 _≃_
-- RECORD
-- isomorphism between sets A and B consists of four things
record _≃_ (A B : Set) : Set where
field
to : A → B -- function from A to B
from : B → A -- function from B to A
from∘to : ∀ (x : A) → from (to x) ≡ x -- evidence asserting 'from' is a left-inverse for 'to'
to∘from : ∀ (y : B) → to (from y) ≡ y -- evidence asserting 'from' is a right-inverse for 'to'
open _≃_ -- makes field names 'to', etc., available without needing to write '_≃_.to'
{-
from ∘ to AND to ∘ from are identities
record declaration behaves similar to single-constructor data declaration
(there are minor differences - see Connectives):
-}
data _≃′_ (A B : Set): Set where
mk-≃′ : ∀ (to : A → B)
→ ∀ (from : B → A)
→ ∀ (from∘to : (∀ (x : A) → from (to x) ≡ x))
→ ∀ (to∘from : (∀ (y : B) → to (from y) ≡ y))
→ A ≃′ B
to′ : ∀ {A B : Set} → (A ≃′ B) → (A → B)
to′ (mk-≃′ f g g∘f f∘g) = f
from′ : ∀ {A B : Set} → (A ≃′ B) → (B → A)
from′ (mk-≃′ f g g∘f f∘g) = g
from∘to′ : ∀ {A B : Set} → (A≃B : A ≃′ B) → (∀ (x : A) → from′ A≃B (to′ A≃B x) ≡ x)
from∘to′ (mk-≃′ f g g∘f f∘g) = g∘f
to∘from′ : ∀ {A B : Set} → (A≃B : A ≃′ B) → (∀ (y : B) → to′ A≃B (from′ A≃B y) ≡ y)
to∘from′ (mk-≃′ f g g∘f f∘g) = f∘g
{-
construct record values via
record
{ to = f
; from = g
; from∘to = g∘f
; to∘from = f∘g
}
corresponds to using the constructor of the corresponding inductive type
mk-≃′ f g g∘f f∘g
------------------------------------------------------------------------------
ISOMORPHISM is an EQUIVALENCE : REFLEXIVE, SYMMETRIC, and TRANSITIVE
-}
-- REFLEXIVE
≃-refl : ∀ {A : Set}
-----
→ A ≃ A
≃-refl =
record
{ to = λ{x → x} -- bind to identity function
; from = λ{y → y} -- ditto
-- refl next is proof since for left inverse, from (to x) simplifies to x, and vice versa
; from∘to = λ{x → refl} -- bound to fun that discards arg; returns refl
; to∘from = λ{y → refl} -- ditto
}
-- SYMMETRIC : swap roles of to/from and from∘to/to∘from
≃-sym : ∀ {A B : Set}
→ A ≃ B
-----
→ B ≃ A
≃-sym A≃B =
record
{ to = from A≃B
; from = to A≃B
; from∘to = to∘from A≃B
; to∘from = from∘to A≃B
}
-- TRANSITIVE : compose to/from and use equational reasoning to combine inverses
≃-trans : ∀ {A B C : Set}
→ A ≃ B
→ B ≃ C
-----
→ A ≃ C
≃-trans A≃B B≃C =
record
{ to = to B≃C ∘ to A≃B
; from = from A≃B ∘ from B≃C
; from∘to = λ{x →
begin
(from A≃B ∘ from B≃C) ((to B≃C ∘ to A≃B) x) ≡⟨⟩
from A≃B (from B≃C (to B≃C (to A≃B x))) ≡⟨ cong (from A≃B) (from∘to B≃C (to A≃B x)) ⟩
from A≃B (to A≃B x) ≡⟨ from∘to A≃B x ⟩
x
∎}
; to∘from = λ{y →
begin
(to B≃C ∘ to A≃B) ((from A≃B ∘ from B≃C) y) ≡⟨⟩
to B≃C (to A≃B (from A≃B (from B≃C y))) ≡⟨ cong (to B≃C) (to∘from A≃B (from B≃C y)) ⟩
to B≃C (from B≃C y) ≡⟨ to∘from B≃C y ⟩
y
∎}
}
{-
------------------------------------------------------------------------------
EQUATIONAL REASONING FOR ISOMORPHISM
Essentially copy previous definition of equality for isomorphism.
Omit the form that corresponds to _≡⟨⟩_,
since simple isomorphisms arise less often than simple equalities
-}
module ≃-Reasoning where
infix 1 ≃-begin_
infixr 2 _≃⟨_⟩_
infix 3 _≃-∎
≃-begin_ : ∀ {A B : Set}
→ A ≃ B
-----
→ A ≃ B
≃-begin A≃B = A≃B
_≃⟨_⟩_ : ∀ (A : Set) {B C : Set}
→ A ≃ B
→ B ≃ C
-----
→ A ≃ C
A ≃⟨ A≃B ⟩ B≃C = ≃-trans A≃B B≃C
_≃-∎ : ∀ (A : Set)
-----
→ A ≃ A
A ≃-∎ = ≃-refl
open ≃-Reasoning
{-
------------------------------------------------------------------------------
EMBEDDING : WEAKENING of ISOMORPHISM : EMBEDDING SHOWS 1ST TYPE INCLUDED IN SECOND
i.e., there is many-to-one correspondence between second type and first
-}
infix 0 _≲_
record _≲_ (A B : Set) : Set where
field
to : A → B
from : B → A
from∘to : ∀ (x : A) → from (to x) ≡ x
open _≲_
{-
same as isomorphism, except it omits 'to∘from' field
- says 'from' is left-inverse for 'to', but not a right-inverse
EMBEDDING IS NOT SYMMETRIC
proofs of REFLEXIVE and TRANSITIVE same as ISOMORPHISM except omitting one unneeded case
-}
-- REFLEXIVE
≲-refl : ∀ {A : Set} → A ≲ A
≲-refl =
record
{ to = λ{x → x}
; from = λ{y → y}
; from∘to = λ{x → refl}
}
-- TRANSITIVE
≲-trans : ∀ {A B C : Set} → A ≲ B → B ≲ C → A ≲ C
≲-trans A≲B B≲C =
record
{ to = λ{x → to B≲C (to A≲B x)}
; from = λ{y → from A≲B (from B≲C y)}
; from∘to = λ{x →
begin
from A≲B (from B≲C (to B≲C (to A≲B x))) ≡⟨ cong (from A≲B) (from∘to B≲C (to A≲B x)) ⟩
from A≲B (to A≲B x) ≡⟨ from∘to A≲B x ⟩
x
∎}
}
{-
weak form of ANTI-SYMMETRY
if two types embed in each other, and embedding functions correspond, they are isomorphic
-}
≲-antisym : ∀ {A B : Set}
→ (A≲B : A ≲ B)
→ (B≲A : B ≲ A)
→ (to A≲B ≡ from B≲A)
→ (from A≲B ≡ to B≲A)
-------------------
→ A ≃ B
≲-antisym A≲B B≲A to≡from from≡to =
record
{ to = to A≲B
; from = from A≲B
; from∘to = from∘to A≲B
; to∘from = λ{y →
begin
to A≲B (from A≲B y) ≡⟨ cong (to A≲B) (cong-app from≡to y) ⟩
to A≲B (to B≲A y) ≡⟨ cong-app to≡from (to B≲A y) ⟩
from B≲A (to B≲A y) ≡⟨ from∘to B≲A y ⟩
y
∎}
}
{-
First three components are copied from the embedding.
The last combines left inverse of B ≲ A with the equivalences of the 'to' and 'from' components
from the two embeddings to obtain the right inverse of the isomorphism.
------------------------------------------------------------------------------
Equational reasoning for embedding
-}
module ≲-Reasoning where
infix 1 ≲-begin_
infixr 2 _≲⟨_⟩_
infix 3 _≲-∎
≲-begin_ : ∀ {A B : Set}
→ A ≲ B
-----
→ A ≲ B
≲-begin A≲B = A≲B
_≲⟨_⟩_ : ∀ (A : Set) {B C : Set}
→ A ≲ B
→ B ≲ C
-----
→ A ≲ C
A ≲⟨ A≲B ⟩ B≲C = ≲-trans A≲B B≲C
_≲-∎ : ∀ (A : Set)
-----
→ A ≲ A
A ≲-∎ = ≲-refl
open ≲-Reasoning
{-
------------------------------------------------------------------------------
Exercise ≃-implies-≲ (practice) Show that every isomorphism implies an embedding. TODO
postulate
≃-implies-≲ : ∀ {A B : Set}
→ A ≃ B
-----
→ A ≲ B
-- Your code goes here
------------------------------------------------------------------------------
Exercise _⇔_ (practice) Define equivalence of propositions TODO
(also known as “if and only if”) as follows:
record _⇔_ (A B : Set) : Set where
field
to : A → B
from : B → A
Show that equivalence is reflexive, symmetric, and transitive.
-- Your code goes here
------------------------------------------------------------------------------
Exercise Bin-embedding (stretch) TODO
Bin and Bin-laws define a datatype Bin of bitstrings representing natural numbers
with functions
to : ℕ → Bin
from : Bin → ℕ
that satisfy
from (to n) ≡ n
Using the above, establish that there is an embedding of ℕ into Bin.
-- Your code goes here
Why do to and from not form an isomorphism?
------------------------------------------------------------------------------
Standard library
import Function using (_∘_)
import Function.Inverse using (_↔_)
import Function.LeftInverse using (_↞_)
The standard library _↔︎_ and _↞_ correspond to our _≃_ and _≲_, respectively,
but those in the standard library are less convenient,
since they depend on a nested record structure
and are parameterised with regard to an arbitrary notion of equivalence.
------------------------------------------------------------------------------
Unicode
This chapter uses the following unicode:
∘ U+2218 RING OPERATOR (\o, \circ, \comp)
λ U+03BB GREEK SMALL LETTER LAMBDA (\lambda, \Gl)
≃ U+2243 ASYMPTOTICALLY EQUAL TO (\~-)
≲ U+2272 LESS-THAN OR EQUIVALENT TO (\<~)
⇔ U+21D4 LEFT RIGHT DOUBLE ARROW (\<=>)
-}
| {
"alphanum_fraction": 0.489564389,
"avg_line_length": 26.3630136986,
"ext": "agda",
"hexsha": "2c2be464e1364b8ca3a116cf4e796be4674138ca",
"lang": "Agda",
"max_forks_count": 8,
"max_forks_repo_forks_event_max_datetime": "2021-09-21T15:58:10.000Z",
"max_forks_repo_forks_event_min_datetime": "2015-04-13T21:40:15.000Z",
"max_forks_repo_head_hexsha": "3dc7abca7ad868316bb08f31c77fbba0d3910225",
"max_forks_repo_licenses": [
"Unlicense"
],
"max_forks_repo_name": "haroldcarr/learn-haskell-coq-ml-etc",
"max_forks_repo_path": "agda/book/Programming_Language_Foundations_in_Agda/x05isomorphism.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "3dc7abca7ad868316bb08f31c77fbba0d3910225",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"Unlicense"
],
"max_issues_repo_name": "haroldcarr/learn-haskell-coq-ml-etc",
"max_issues_repo_path": "agda/book/Programming_Language_Foundations_in_Agda/x05isomorphism.agda",
"max_line_length": 99,
"max_stars_count": 36,
"max_stars_repo_head_hexsha": "3dc7abca7ad868316bb08f31c77fbba0d3910225",
"max_stars_repo_licenses": [
"Unlicense"
],
"max_stars_repo_name": "haroldcarr/learn-haskell-coq-ml-etc",
"max_stars_repo_path": "agda/book/Programming_Language_Foundations_in_Agda/x05isomorphism.agda",
"max_stars_repo_stars_event_max_datetime": "2021-07-30T06:55:03.000Z",
"max_stars_repo_stars_event_min_datetime": "2015-01-29T14:37:15.000Z",
"num_tokens": 4030,
"size": 11547
} |
open import Common.Prelude
open import Common.Reflection
module TermSplicingOutOfScope where
f : Set → Set → Set → Set
f x y z = unquote (give (var 3 []))
| {
"alphanum_fraction": 0.7261146497,
"avg_line_length": 19.625,
"ext": "agda",
"hexsha": "f60b770c6dd6a8bee4350141e99aadb385e07aad",
"lang": "Agda",
"max_forks_count": 371,
"max_forks_repo_forks_event_max_datetime": "2022-03-30T19:00:30.000Z",
"max_forks_repo_forks_event_min_datetime": "2015-01-03T14:04:08.000Z",
"max_forks_repo_head_hexsha": "231d6ad8e77b67ff8c4b1cb35a6c31ccd988c3e9",
"max_forks_repo_licenses": [
"BSD-3-Clause"
],
"max_forks_repo_name": "Agda-zh/agda",
"max_forks_repo_path": "test/Fail/TermSplicingOutOfScope.agda",
"max_issues_count": 4066,
"max_issues_repo_head_hexsha": "ed8ac6f4062ea8a20fa0f62d5db82d4e68278338",
"max_issues_repo_issues_event_max_datetime": "2022-03-31T21:14:49.000Z",
"max_issues_repo_issues_event_min_datetime": "2015-01-10T11:24:51.000Z",
"max_issues_repo_licenses": [
"BSD-3-Clause"
],
"max_issues_repo_name": "shlevy/agda",
"max_issues_repo_path": "test/Fail/TermSplicingOutOfScope.agda",
"max_line_length": 35,
"max_stars_count": 1989,
"max_stars_repo_head_hexsha": "ed8ac6f4062ea8a20fa0f62d5db82d4e68278338",
"max_stars_repo_licenses": [
"BSD-3-Clause"
],
"max_stars_repo_name": "shlevy/agda",
"max_stars_repo_path": "test/Fail/TermSplicingOutOfScope.agda",
"max_stars_repo_stars_event_max_datetime": "2022-03-30T18:20:48.000Z",
"max_stars_repo_stars_event_min_datetime": "2015-01-09T23:51:16.000Z",
"num_tokens": 44,
"size": 157
} |
{- Byzantine Fault Tolerant Consensus Verification in Agda, version 0.9.
Copyright (c) 2020, 2021, Oracle and/or its affiliates.
Licensed under the Universal Permissive License v 1.0 as shown at https://opensource.oracle.com/licenses/upl
-}
open import Optics.All
open import LibraBFT.Prelude
open import LibraBFT.Base.ByteString
open import LibraBFT.Base.PKCS
open import LibraBFT.Base.Types
open import LibraBFT.Hash
open import LibraBFT.Impl.Base.Types
open import LibraBFT.Impl.Consensus.Types
open import LibraBFT.Impl.Util.Crypto
open import LibraBFT.Impl.Util.Util
open import LibraBFT.Abstract.Types.EpochConfig UID NodeId
-- This is a minimal/fake example handler that obeys the VotesOnce rule, enabling us to start
-- exploring how we express the algorithm and prove properties about it. It simply sends a vote for
-- 1 + its LatestVotedRound, and increments its LatestVotedRound. It is called RoundManager for
-- historical reasons, because this what a previous version of LibraBFT called its main handler;
-- this will be updated when we move towards modeling a more recent implementation.
module LibraBFT.Impl.Consensus.RoundManager where
open RWST-do
processCommitM : LedgerInfoWithSignatures → LBFT (List ExecutedBlock)
processCommitM finalityProof = pure []
fakeAuthor : Author
fakeAuthor = 0
fakeBlockInfo : Epoch → Round → ProposalMsg → BlockInfo
fakeBlockInfo eid rnd pm = BlockInfo∙new eid rnd (pm ^∙ pmProposal ∙ bId)
fakeLedgerInfo : BlockInfo → ProposalMsg → LedgerInfo
fakeLedgerInfo bi pm = LedgerInfo∙new bi (pm ^∙ pmProposal ∙ bId)
postulate -- TODO-1: these are temporary scaffolding for the fake implementation
fakeSK : SK
fakeSig : Signature
processProposalMsg : Instant → ProposalMsg → LBFT Unit
processProposalMsg inst pm = do
st ← get
xx ← use rmHighestQC -- Not used; just a demonstration that our RoundManager-specific "use" works
modify' rmHighestQC xx -- Similarly for modify'
let RoundManager∙new rm rmc rmw = st
𝓔 = α-EC (rm , rmc)
e = rm ^∙ rmEpoch
nr = suc (rm ^∙ rmLastVotedRound)
uv = Vote∙new
(VoteData∙new (fakeBlockInfo e nr pm) (fakeBlockInfo e 0 pm))
fakeAuthor
(fakeLedgerInfo (fakeBlockInfo e nr pm) pm)
fakeSig
nothing
sv = record uv { ₋vSignature = sign ⦃ sig-Vote ⦄ uv fakeSK}
bt = rmw ^∙ (lBlockTree 𝓔)
si = SyncInfo∙new (₋btHighestQuorumCert bt) (₋btHighestCommitCert bt)
rm' = rm [ rmLastVotedRound := nr ]
st' = RoundManager∙new rm' (RoundManagerEC-correct-≡ (₋rmEC st) rm' refl rmc)
(subst RoundManagerWithEC (α-EC-≡ rm rm' refl refl rmc) rmw)
put st'
tell1 (SendVote (VoteMsg∙new sv si) (fakeAuthor ∷ []))
pure unit
processVote : Instant → VoteMsg → LBFT Unit
processVote now msg = pure unit
| {
"alphanum_fraction": 0.6973193078,
"avg_line_length": 40.9305555556,
"ext": "agda",
"hexsha": "690a0058da77c76813a7dcddc5e8c5e01becf269",
"lang": "Agda",
"max_forks_count": null,
"max_forks_repo_forks_event_max_datetime": null,
"max_forks_repo_forks_event_min_datetime": null,
"max_forks_repo_head_hexsha": "71aa2168e4875ffdeece9ba7472ee3cee5fa9084",
"max_forks_repo_licenses": [
"UPL-1.0"
],
"max_forks_repo_name": "cwjnkins/bft-consensus-agda",
"max_forks_repo_path": "LibraBFT/Impl/Consensus/RoundManager.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "71aa2168e4875ffdeece9ba7472ee3cee5fa9084",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"UPL-1.0"
],
"max_issues_repo_name": "cwjnkins/bft-consensus-agda",
"max_issues_repo_path": "LibraBFT/Impl/Consensus/RoundManager.agda",
"max_line_length": 111,
"max_stars_count": null,
"max_stars_repo_head_hexsha": "71aa2168e4875ffdeece9ba7472ee3cee5fa9084",
"max_stars_repo_licenses": [
"UPL-1.0"
],
"max_stars_repo_name": "cwjnkins/bft-consensus-agda",
"max_stars_repo_path": "LibraBFT/Impl/Consensus/RoundManager.agda",
"max_stars_repo_stars_event_max_datetime": null,
"max_stars_repo_stars_event_min_datetime": null,
"num_tokens": 832,
"size": 2947
} |
open import Agda.Builtin.Nat
record _×_ (A B : Set) : Set where
constructor _,_
field fst : A
snd : B
open _×_
Δ : ∀ {A} → A → A × A
Δ x = x , x
foo : Nat → Nat
foo n = let x , y = Δ n in x + y
bar : Nat → Nat
bar n = let _!_ : Nat → Nat → Nat
x ! y = 2 * x + y
in n ! n
| {
"alphanum_fraction": 0.4724919094,
"avg_line_length": 14.7142857143,
"ext": "agda",
"hexsha": "44ed0696bdcd9ee52ee58882417bee83a65e76cf",
"lang": "Agda",
"max_forks_count": 371,
"max_forks_repo_forks_event_max_datetime": "2022-03-30T19:00:30.000Z",
"max_forks_repo_forks_event_min_datetime": "2015-01-03T14:04:08.000Z",
"max_forks_repo_head_hexsha": "7f58030124fa99dfbf8db376659416f3ad8384de",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "cruhland/agda",
"max_forks_repo_path": "test/Succeed/Issue917.agda",
"max_issues_count": 4066,
"max_issues_repo_head_hexsha": "7f58030124fa99dfbf8db376659416f3ad8384de",
"max_issues_repo_issues_event_max_datetime": "2022-03-31T21:14:49.000Z",
"max_issues_repo_issues_event_min_datetime": "2015-01-10T11:24:51.000Z",
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "cruhland/agda",
"max_issues_repo_path": "test/Succeed/Issue917.agda",
"max_line_length": 34,
"max_stars_count": 1989,
"max_stars_repo_head_hexsha": "7f58030124fa99dfbf8db376659416f3ad8384de",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "cruhland/agda",
"max_stars_repo_path": "test/Succeed/Issue917.agda",
"max_stars_repo_stars_event_max_datetime": "2022-03-30T18:20:48.000Z",
"max_stars_repo_stars_event_min_datetime": "2015-01-09T23:51:16.000Z",
"num_tokens": 124,
"size": 309
} |
open import Data.Empty
open import Data.Maybe
open import Data.Product
open import Data.Sum
open import AEff
open import EffectAnnotations
open import Types
open import Relation.Binary.PropositionalEquality hiding ([_])
open import Relation.Nullary
open import Relation.Nullary.Negation
module AwaitingComputations where
-- COMPUTATIONS THAT ARE TEMPORARILY STUCK DUE TO AWAITING FOR A PARTICULAR PROMISE
data _⧗_ {Γ : Ctx} {X : VType} (x : ⟨ X ⟩ ∈ Γ) : {C : CType} → Γ ⊢M⦂ C → Set where
await : {C : CType}
{M : Γ ∷ X ⊢M⦂ C} →
-------------------------
x ⧗ (await (` x) until M)
let-in : {X Y : VType}
{o : O}
{i : I}
{M : Γ ⊢M⦂ X ! (o , i)}
{N : Γ ∷ X ⊢M⦂ Y ! (o , i)} →
x ⧗ M →
-----------------------------
x ⧗ (let= M `in N)
interrupt : {X : VType}
{o : O}
{i : I}
{op : Σₛ}
{V : Γ ⊢V⦂ ``(payload op)}
{M : Γ ⊢M⦂ X ! (o , i)} →
x ⧗ M →
-------------------------
x ⧗ (↓ op V M)
coerce : {X : VType}
{o o' : O}
{i i' : I}
{p : o ⊑ₒ o'}
{q : i ⊑ᵢ i'}
{M : Γ ⊢M⦂ X ! (o , i)} →
x ⧗ M →
-------------------------
x ⧗ (coerce p q M)
| {
"alphanum_fraction": 0.3770147162,
"avg_line_length": 26.9245283019,
"ext": "agda",
"hexsha": "9c54c342963a74a5ff3113476465d5e453edbef3",
"lang": "Agda",
"max_forks_count": null,
"max_forks_repo_forks_event_max_datetime": null,
"max_forks_repo_forks_event_min_datetime": null,
"max_forks_repo_head_hexsha": "71ebed9f90a3eb37ae6cd209457bae23a4d122d1",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "danelahman/aeff-agda",
"max_forks_repo_path": "AwaitingComputations.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "71ebed9f90a3eb37ae6cd209457bae23a4d122d1",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "danelahman/aeff-agda",
"max_issues_repo_path": "AwaitingComputations.agda",
"max_line_length": 83,
"max_stars_count": 4,
"max_stars_repo_head_hexsha": "71ebed9f90a3eb37ae6cd209457bae23a4d122d1",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "danelahman/aeff-agda",
"max_stars_repo_path": "AwaitingComputations.agda",
"max_stars_repo_stars_event_max_datetime": "2021-03-22T22:48:48.000Z",
"max_stars_repo_stars_event_min_datetime": "2020-07-17T00:15:00.000Z",
"num_tokens": 444,
"size": 1427
} |
{-# OPTIONS --without-K --safe #-}
module Dodo.Binary.Immediate where
-- Stdlib imports
import Relation.Binary.PropositionalEquality as Eq
open Eq using (_≡_; _≢_; refl; subst) renaming (sym to ≡-sym)
open import Level using (Level; _⊔_)
open import Function using (_∘_; flip)
open import Data.Empty using (⊥-elim)
open import Data.Product using (_×_; _,_; proj₁; proj₂; ∃-syntax)
open import Data.Sum using (_⊎_; inj₁; inj₂)
open import Relation.Nullary using (¬_)
open import Relation.Unary using (Pred)
open import Relation.Binary using (Rel; REL)
open import Relation.Binary using (IsStrictTotalOrder; Irreflexive; Trichotomous)
open import Relation.Binary using (Transitive)
open import Relation.Binary using (Tri; tri<; tri≈; tri>)
open import Relation.Binary.Construct.Closure.Transitive using (TransClosure; [_]; _∷_; _∷ʳ_; _++_)
-- Local imports
open import Dodo.Unary.Equality
open import Dodo.Unary.Unique
open import Dodo.Binary.Equality
open import Dodo.Binary.Transitive
open import Dodo.Binary.Functional
open import Dodo.Binary.Filter
open import Dodo.Binary.Domain
-- # Definitions #
-- | The immediate relation over the given (order) relation
immediate : ∀ {a ℓ : Level} {A : Set a}
→ Rel A ℓ
-------------
→ Rel A (a ⊔ ℓ)
immediate r x y = r x y × ¬ (∃[ z ] r x z × TransClosure r z y)
-- A more conventional definitions is:
-- immediate r x y = r x y × (¬ ∃ λ{z → r x z × r z y})
-- which is identical to this one when r is Transitive
Immediate : ∀ {a ℓ : Level} {A : Set a}
→ Rel A ℓ
→ Set (a ⊔ ℓ)
-- For some reason, x and y have to be /explicit/. Otherwise, Agda complains about some
-- of Immediate's uses. Unsure why.
Immediate {A = A} r = ∀ (x y : A) → r x y → ¬ (∃[ z ] r x z × TransClosure r z y)
-- # Operations #
imm-flip : ∀ {a ℓ : Level} {A : Set a}
→ {R : Rel A ℓ} {x y : A}
→ immediate R x y
→ immediate (flip R) y x
imm-flip {R = R} {x} {y} (Rxy , ¬∃z) = (Rxy , lemma)
where
⁺-invert : {a ℓ : Level} {A : Set a} {R : Rel A ℓ} {x y : A}
→ {z : A} → R x z → TransClosure R z y
→ ∃[ q ] (TransClosure R x q × R q y)
⁺-invert {z = z} Rxz [ Rzy ] = (z , [ Rxz ] , Rzy)
⁺-invert {z = z} Rxz ( Rzq ∷ R⁺qy ) with ⁺-invert Rzq R⁺qy
... | v , R⁺zv , Rvy = (v , Rxz ∷ R⁺zv , Rvy)
lemma : ¬ (∃[ z ] (flip R y z × TransClosure (flip R) z x))
lemma (z , flipRyz , flipR⁺zx) =
let (q , R⁺yq , Rqx) = ⁺-invert flipRyz flipR⁺zx
in ¬∃z (q , Rqx , ⁺-flip R⁺yq)
-- # Properties #
module _ {a ℓ : Level} {A : Set a} {R : Rel A ℓ} where
imm-imm : Immediate (immediate R)
imm-imm _ _ (Rxy , ¬∃z) (z , (Rxz , ¬∃w) , [immR]⁺xy) = ¬∃z (z , Rxz , ⁺-map _ proj₁ [immR]⁺xy)
imm-⊆₂ : immediate R ⊆₂ R
imm-⊆₂ = ⊆: λ{_ _ → proj₁}
module _ {a ℓ₁ ℓ₂ : Level} {A : Set a} {_≈_ : Rel A ℓ₁} {_<_ : Rel A ℓ₂} where
imm-uniqueˡ : Trichotomous _≈_ _<_ → {z : A} → Unique₁ _≈_ λ{τ → immediate _<_ τ z}
imm-uniqueˡ triR {z} {x} {y} (Rxz , ¬∃y) (Ryz , ¬∃x) with triR x y
... | tri< Rxy x≉y ¬Ryx = ⊥-elim (¬∃y (y , Rxy , [ Ryz ]))
... | tri≈ ¬Rxy x≈y ¬Ryx = x≈y
... | tri> ¬Rxy x≉y Ryx = ⊥-elim (¬∃x (x , Ryx , [ Rxz ]))
imm-uniqueʳ : Trichotomous _≈_ _<_ → {x : A} → Unique₁ _≈_ (immediate _<_ x)
imm-uniqueʳ triR {x} {y} {z} (Rxy , ¬∃z) (Rxz , ¬∃y) with triR y z
... | tri< Ryz y≈z ¬Rzy = ⊥-elim (¬∃y (y , Rxy , [ Ryz ]))
... | tri≈ ¬Ryz y≈z ¬Rzy = y≈z
... | tri> ¬Ryz y≈z Rzy = ⊥-elim (¬∃z (z , Rxz , [ Rzy ]))
module _ {a ℓ₁ ℓ₂ : Level} {A : Set a} {≈ : Rel A ℓ₁} {< : Rel A ℓ₂} where
-- immediate < x y → immediate < x z → y ≈ z
imm-func : IsStrictTotalOrder ≈ < → Functional ≈ (immediate <)
imm-func sto x y₁ y₂ (x<y₁ , ¬∃z[x<z×z<y₁]) (x<y₂ , ¬∃z[x<z×z<y₂])
with IsStrictTotalOrder.compare sto y₁ y₂
... | tri< y₁<y₂ _ _ = ⊥-elim (¬∃z[x<z×z<y₂] (y₁ , x<y₁ , [ y₁<y₂ ]))
... | tri≈ _ y₁≈y₂ _ = y₁≈y₂
... | tri> _ _ y₂<y₁ = ⊥-elim (¬∃z[x<z×z<y₁] (y₂ , x<y₂ , [ y₂<y₁ ]))
module _ {a ℓ₁ ℓ₂ : Level} {A : Set a} {P : Pred A ℓ₁} {R : Rel A ℓ₂} where
imm-filter-⊆₂ : filter-rel P (immediate R) ⊆₂ immediate (filter-rel P R)
imm-filter-⊆₂ = ⊆: lemma
where
lemma : filter-rel P (immediate R) ⊆₂' immediate (filter-rel P R)
lemma (with-pred x Px) (with-pred y Py) (Rxy , ¬∃z) = Rxy , ¬∃z'
where
¬∃z' : ¬ (∃[ z ] (filter-rel P R (with-pred x Px) z × TransClosure (filter-rel P R) z (with-pred y Py)))
¬∃z' (with-pred z Pz , Rxz , fR⁺zy) = ¬∃z (z , Rxz , ⁺-strip-filter fR⁺zy)
module _ {a ℓ : Level} {A : Set a} {R : Rel A ℓ} where
immediate⁺ : Immediate R → R ⇔₂ immediate (TransClosure R)
immediate⁺ immR = ⇔: ⊆-proof ⊇-proof
where
⊆-proof : R ⊆₂' immediate (TransClosure R)
⊆-proof x y xRy = ([ xRy ] , lemma x y xRy)
where
lemma : (x y : A) → R x y → ¬ (∃[ z ] TransClosure R x z × TransClosure (TransClosure R) z y)
lemma x y xRy (z , [ xRz ] , zR⁺y) =
immR x y xRy (z , xRz , ⇔₂-apply-⊇₂ ⁺-idem zR⁺y)
lemma x y xRy (z , _∷_ {_} {w} xRw wR⁺z , zR⁺y) =
immR x y xRy (w , xRw , ⇔₂-apply-⊇₂ ⁺-idem (wR⁺z ∷ zR⁺y))
⊇-proof : immediate (TransClosure R) ⊆₂' R
⊇-proof x y ([ x∼y ] , ¬∃z) = x∼y
⊇-proof x y (_∷_ {_} {w} x∼w wR⁺y , ¬∃z) = ⊥-elim (¬∃z (w , [ x∼w ] , [ wR⁺y ]))
trans-imm⁺-⊆ : Transitive R → TransClosure (immediate R) ⊆₂ R
trans-imm⁺-⊆ transR = ⊆: lemma
where
lemma : TransClosure (immediate R) ⊆₂' R
lemma x y [ R[xy] ] = proj₁ R[xy]
lemma x y (_∷_ {_} {z} R[xz] R⁺[zy]) = transR (proj₁ R[xz]) (lemma z y R⁺[zy])
imm-udr-⊆₁ : udr (immediate R) ⊆₁ udr R
imm-udr-⊆₁ = ⊆: lemma
where
lemma : udr (immediate R) ⊆₁' udr R
lemma _ (inj₁ (y , Rxy , ¬∃z)) = inj₁ (y , Rxy)
lemma _ (inj₂ (x , Rxy , ¬∃z)) = inj₂ (x , Rxy)
| {
"alphanum_fraction": 0.5584892464,
"avg_line_length": 36.8967741935,
"ext": "agda",
"hexsha": "801e6b37d2a29e317c31eef7d4df9cf133c0e04b",
"lang": "Agda",
"max_forks_count": null,
"max_forks_repo_forks_event_max_datetime": null,
"max_forks_repo_forks_event_min_datetime": null,
"max_forks_repo_head_hexsha": "376f0ccee1e1aa31470890e494bcb534324f598a",
"max_forks_repo_licenses": [
"BSD-3-Clause"
],
"max_forks_repo_name": "sourcedennis/agda-dodo",
"max_forks_repo_path": "src/Dodo/Binary/Immediate.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "376f0ccee1e1aa31470890e494bcb534324f598a",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"BSD-3-Clause"
],
"max_issues_repo_name": "sourcedennis/agda-dodo",
"max_issues_repo_path": "src/Dodo/Binary/Immediate.agda",
"max_line_length": 110,
"max_stars_count": null,
"max_stars_repo_head_hexsha": "376f0ccee1e1aa31470890e494bcb534324f598a",
"max_stars_repo_licenses": [
"BSD-3-Clause"
],
"max_stars_repo_name": "sourcedennis/agda-dodo",
"max_stars_repo_path": "src/Dodo/Binary/Immediate.agda",
"max_stars_repo_stars_event_max_datetime": null,
"max_stars_repo_stars_event_min_datetime": null,
"num_tokens": 2490,
"size": 5719
} |
module Signature where
open import Data.Product renaming (Σ to ⨿)
open import Function
open import Relation.Binary.PropositionalEquality using (_≡_; refl; subst)
open import Function
open import Data.Empty
open import Data.Unit hiding (_≤_)
open import Data.Product as Prod renaming (Σ to ⨿)
open import Data.Nat as Nat
open import Data.Sum as Sum
record Sig : Set₁ where
field
∥_∥ : Set
ar : ∥_∥ → Set
open Sig public
-- | Extension of signature Σ, on objects
⟪_⟫ : Sig → Set → Set
⟪ Σ ⟫ X = ⨿ ∥ Σ ∥ λ f → (ar Σ f → X)
-- | Extension of signature Σ, on morphisms
⟪_⟫₁ : (Σ : Sig) {A B : Set} → (A → B) → ⟪ Σ ⟫ A → ⟪ Σ ⟫ B
⟪_⟫₁ Σ f (s , α) = (s , f ∘ α)
-- | Lift ⟪ Σ ⟫ to relations
sig-lift : {Σ : Sig} {X : Set} (R : X → X → Set) (x y : ⟪ Σ ⟫ X) → Set
sig-lift {Σ} R (f , α) (g , β) =
⨿ (f ≡ g) λ p → ∀ {i} → R (α i) (β (subst (Sig.ar Σ) p i))
| {
"alphanum_fraction": 0.5898030127,
"avg_line_length": 27.8387096774,
"ext": "agda",
"hexsha": "563047a83f084a5951b72f5efb92f83e9bed47ad",
"lang": "Agda",
"max_forks_count": null,
"max_forks_repo_forks_event_max_datetime": null,
"max_forks_repo_forks_event_min_datetime": null,
"max_forks_repo_head_hexsha": "8fc7a6cd878f37f9595124ee8dea62258da28aa4",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "hbasold/Sandbox",
"max_forks_repo_path": "LP2/Signature.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "8fc7a6cd878f37f9595124ee8dea62258da28aa4",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "hbasold/Sandbox",
"max_issues_repo_path": "LP2/Signature.agda",
"max_line_length": 74,
"max_stars_count": null,
"max_stars_repo_head_hexsha": "8fc7a6cd878f37f9595124ee8dea62258da28aa4",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "hbasold/Sandbox",
"max_stars_repo_path": "LP2/Signature.agda",
"max_stars_repo_stars_event_max_datetime": null,
"max_stars_repo_stars_event_min_datetime": null,
"num_tokens": 354,
"size": 863
} |
module Lattice where
open import Prelude
open import PartialOrder as PO
open import SemiLattice as SL
import Chain
open POrder using (Dual)
record Lattice (A : Set) : Set1 where
field
sl : SemiLattice A
_⊔_ : A -> A -> A
prf : IsSemiLattice (Dual (SemiLat.po sl)) _⊔_
module Lat {A : Set}(L : Lattice A) where
private
module LL = Lattice L
module SLL = SemiLat LL.sl
private
sl' : SemiLattice A
sl' = record { po = Dual SLL.po; _⊓_ = LL._⊔_; prf = LL.prf }
module SLL' = SemiLat sl'
hiding ( Monotone
; Antitone
; _==_; ==-refl; ==-sym; ==-trans
; po
)
renaming ( _≤_ to _≥_
; ≤-refl to ≥-refl
; ≤-trans to ≥-trans
; ≤-antisym to ≥-antisym
; ==≤-L to ==≥-R
; ==≤-R to ==≥-L
; _⊓_ to _⊔_
; ⊓-lbL to ⊔-ubL
; ⊓-lbR to ⊔-ubR
; ⊓-glb to ⊔-lub
; ⊓-commute to ⊔-commute
; ⊓-assoc to ⊔-assoc
; ⊓-idem to ⊔-idem
; ≤⊓-L to ≥⊔-L
; ≤⊓-R to ≥⊔-R
; ⊓-monotone-R to ⊔-monotone-R
; ⊓-monotone-L to ⊔-monotone-L
; ≤⊓-compat to ≥⊔-compat
; ⊓-cong to ⊔-cong
; ⊓-cong-L to ⊔-cong-L
; ⊓-cong-R to ⊔-cong-R
)
open SLL public
open SLL' public
DualLattice : Lattice A
DualLattice = record { sl = sl'; _⊔_ = _⊓_; prf = SemiLattice.prf LL.sl }
module MeetJoin {A : Set}(L : Lattice A) where
private module L = Lat L
open L
open module C== = Chain _==_ (\x -> ==-refl) (\x y z -> ==-trans)
-- Experiment with very explicit proof
⊓⊔-absorb-LL = \{x y} ->
(x ⊓ (x ⊔ y)) == x from
≤-antisym
((x ⊓ (x ⊔ y)) ≤ x from ⊓-lbL)
(x ≤ (x ⊓ (x ⊔ y)) from
⊓-glb (x ≤ x from ≤-refl)
(x ≤ (x ⊔ y) from ⊔-ubL)
)
⊓⊔-eq : forall {x y} -> (x ⊓ y) == (x ⊔ y) -> x == y
⊓⊔-eq {x}{y} p =
chain> x
=== x ⊓ (x ⊔ y) by ==-sym ⊓⊔-absorb-LL
=== x ⊓ (x ⊓ y) by ==-sym (⊓-cong-R p)
=== (x ⊓ x) ⊓ y by {!!} -- ⊓-assoc
=== x ⊓ y by ⊓-cong-L ⊓-idem
=== y ⊓ x by ⊓-commute
=== (y ⊓ y) ⊓ x by ⊓-cong-L (==-sym ⊓-idem)
=== y ⊓ (y ⊓ x) by ==-sym ⊓-assoc
=== y ⊓ (x ⊓ y) by ⊓-cong-R ⊓-commute
=== y ⊓ (x ⊔ y) by {! !} -- ⊓-cong-R p
=== y ⊓ (y ⊔ x) by ⊓-cong-R ⊔-commute
=== y by ⊓⊔-absorb-LL
module JoinMeet {A : Set}(L : Lattice A) =
MeetJoin (Lat.DualLattice L)
hiding (⊓⊔-eq)
renaming (⊓⊔-absorb-LL to ⊔⊓-absorb-LL)
| {
"alphanum_fraction": 0.4041873669,
"avg_line_length": 29.0515463918,
"ext": "agda",
"hexsha": "6d9aa14c5e011d56c1249b3ac8e9e12cc60e1585",
"lang": "Agda",
"max_forks_count": null,
"max_forks_repo_forks_event_max_datetime": null,
"max_forks_repo_forks_event_min_datetime": null,
"max_forks_repo_head_hexsha": "70c8a575c46f6a568c7518150a1a64fcd03aa437",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "masondesu/agda",
"max_forks_repo_path": "examples/outdated-and-incorrect/lattice/Lattice.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "70c8a575c46f6a568c7518150a1a64fcd03aa437",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "masondesu/agda",
"max_issues_repo_path": "examples/outdated-and-incorrect/lattice/Lattice.agda",
"max_line_length": 75,
"max_stars_count": 1,
"max_stars_repo_head_hexsha": "aa10ae6a29dc79964fe9dec2de07b9df28b61ed5",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "asr/agda-kanso",
"max_stars_repo_path": "examples/outdated-and-incorrect/lattice/Lattice.agda",
"max_stars_repo_stars_event_max_datetime": "2019-11-27T04:41:05.000Z",
"max_stars_repo_stars_event_min_datetime": "2019-11-27T04:41:05.000Z",
"num_tokens": 1134,
"size": 2818
} |
open import Agda.Builtin.Nat
record R : Set₁ where
field f : Nat
open R ⦃ ... ⦄
foo : Nat → R
foo n .f = {!n!} -- C-c C-c makes clause disappear
| {
"alphanum_fraction": 0.6026490066,
"avg_line_length": 13.7272727273,
"ext": "agda",
"hexsha": "b94844107dde31b5030b529b35576e8c68223177",
"lang": "Agda",
"max_forks_count": 371,
"max_forks_repo_forks_event_max_datetime": "2022-03-30T19:00:30.000Z",
"max_forks_repo_forks_event_min_datetime": "2015-01-03T14:04:08.000Z",
"max_forks_repo_head_hexsha": "cc026a6a97a3e517bb94bafa9d49233b067c7559",
"max_forks_repo_licenses": [
"BSD-2-Clause"
],
"max_forks_repo_name": "cagix/agda",
"max_forks_repo_path": "test/interaction/Issue4998.agda",
"max_issues_count": 4066,
"max_issues_repo_head_hexsha": "cc026a6a97a3e517bb94bafa9d49233b067c7559",
"max_issues_repo_issues_event_max_datetime": "2022-03-31T21:14:49.000Z",
"max_issues_repo_issues_event_min_datetime": "2015-01-10T11:24:51.000Z",
"max_issues_repo_licenses": [
"BSD-2-Clause"
],
"max_issues_repo_name": "cagix/agda",
"max_issues_repo_path": "test/interaction/Issue4998.agda",
"max_line_length": 50,
"max_stars_count": 1989,
"max_stars_repo_head_hexsha": "cc026a6a97a3e517bb94bafa9d49233b067c7559",
"max_stars_repo_licenses": [
"BSD-2-Clause"
],
"max_stars_repo_name": "cagix/agda",
"max_stars_repo_path": "test/interaction/Issue4998.agda",
"max_stars_repo_stars_event_max_datetime": "2022-03-30T18:20:48.000Z",
"max_stars_repo_stars_event_min_datetime": "2015-01-09T23:51:16.000Z",
"num_tokens": 57,
"size": 151
} |
{-# OPTIONS --safe #-}
module Cubical.HITs.Susp.Properties where
open import Cubical.Foundations.Prelude
open import Cubical.Foundations.HLevels
open import Cubical.Foundations.Isomorphism
open import Cubical.Foundations.Equiv
open import Cubical.Foundations.Path
open import Cubical.Foundations.Pointed
open import Cubical.Foundations.Pointed.Homogeneous
open import Cubical.Foundations.GroupoidLaws
open import Cubical.Data.Bool
open import Cubical.Data.Sigma
open import Cubical.HITs.Join
open import Cubical.HITs.Susp.Base
open import Cubical.Homotopy.Loopspace
private
variable
ℓ : Level
open Iso
Susp-iso-joinBool : ∀ {ℓ} {A : Type ℓ} → Iso (Susp A) (join A Bool)
fun Susp-iso-joinBool north = inr true
fun Susp-iso-joinBool south = inr false
fun Susp-iso-joinBool (merid a i) = (sym (push a true) ∙ push a false) i
inv Susp-iso-joinBool (inr true ) = north
inv Susp-iso-joinBool (inr false) = south
inv Susp-iso-joinBool (inl _) = north
inv Susp-iso-joinBool (push a true i) = north
inv Susp-iso-joinBool (push a false i) = merid a i
rightInv Susp-iso-joinBool (inr true ) = refl
rightInv Susp-iso-joinBool (inr false) = refl
rightInv Susp-iso-joinBool (inl a) = sym (push a true)
rightInv Susp-iso-joinBool (push a true i) j = push a true (i ∨ ~ j)
rightInv Susp-iso-joinBool (push a false i) j
= hcomp (λ k → λ { (i = i0) → push a true (~ j)
; (i = i1) → push a false k
; (j = i1) → push a false (i ∧ k) })
(push a true (~ i ∧ ~ j))
leftInv Susp-iso-joinBool north = refl
leftInv Susp-iso-joinBool south = refl
leftInv (Susp-iso-joinBool {A = A}) (merid a i) j
= hcomp (λ k → λ { (i = i0) → transp (λ _ → Susp A) (k ∨ j) north
; (i = i1) → transp (λ _ → Susp A) (k ∨ j) (merid a k)
; (j = i1) → merid a (i ∧ k) })
(transp (λ _ → Susp A) j north)
Susp≃joinBool : ∀ {ℓ} {A : Type ℓ} → Susp A ≃ join A Bool
Susp≃joinBool = isoToEquiv Susp-iso-joinBool
Susp≡joinBool : ∀ {ℓ} {A : Type ℓ} → Susp A ≡ join A Bool
Susp≡joinBool = isoToPath Susp-iso-joinBool
congSuspIso : ∀ {ℓ} {A B : Type ℓ} → Iso A B → Iso (Susp A) (Susp B)
fun (congSuspIso is) = suspFun (fun is)
inv (congSuspIso is) = suspFun (inv is)
rightInv (congSuspIso is) north = refl
rightInv (congSuspIso is) south = refl
rightInv (congSuspIso is) (merid a i) j = merid (rightInv is a j) i
leftInv (congSuspIso is) north = refl
leftInv (congSuspIso is) south = refl
leftInv (congSuspIso is) (merid a i) j = merid (leftInv is a j) i
congSuspEquiv : ∀ {ℓ} {A B : Type ℓ} → A ≃ B → Susp A ≃ Susp B
congSuspEquiv {ℓ} {A} {B} h = isoToEquiv (congSuspIso (equivToIso h))
suspToPropElim : ∀ {ℓ ℓ'} {A : Type ℓ} {B : Susp A → Type ℓ'} (a : A)
→ ((x : Susp A) → isProp (B x))
→ B north
→ (x : Susp A) → B x
suspToPropElim a isProp Bnorth north = Bnorth
suspToPropElim {B = B} a isProp Bnorth south = subst B (merid a) Bnorth
suspToPropElim {B = B} a isProp Bnorth (merid a₁ i) =
isOfHLevel→isOfHLevelDep 1 isProp Bnorth (subst B (merid a) Bnorth) (merid a₁) i
suspToPropElim2 : ∀ {ℓ ℓ'} {A : Type ℓ} {B : Susp A → Susp A → Type ℓ'} (a : A)
→ ((x y : Susp A) → isProp (B x y))
→ B north north
→ (x y : Susp A) → B x y
suspToPropElim2 _ _ Bnorth north north = Bnorth
suspToPropElim2 {B = B} a _ Bnorth north south = subst (B north) (merid a) Bnorth
suspToPropElim2 {B = B} a isprop Bnorth north (merid x i) =
isProp→PathP (λ i → isprop north (merid x i))
Bnorth (subst (B north) (merid a) Bnorth) i
suspToPropElim2 {B = B} a _ Bnorth south north = subst (λ x → B x north) (merid a) Bnorth
suspToPropElim2 {B = B} a _ Bnorth south south = subst (λ x → B x x) (merid a) Bnorth
suspToPropElim2 {B = B} a isprop Bnorth south (merid x i) =
isProp→PathP (λ i → isprop south (merid x i))
(subst (λ x → B x north) (merid a) Bnorth)
(subst (λ x → B x x) (merid a) Bnorth) i
suspToPropElim2 {B = B} a isprop Bnorth (merid x i) north =
isProp→PathP (λ i → isprop (merid x i) north)
Bnorth (subst (λ x → B x north) (merid a) Bnorth) i
suspToPropElim2 {B = B} a isprop Bnorth (merid x i) south =
isProp→PathP (λ i → isprop (merid x i) south)
(subst (B north) (merid a) Bnorth)
(subst (λ x → B x x) (merid a) Bnorth) i
suspToPropElim2 {B = B} a isprop Bnorth (merid x i) (merid y j) =
isSet→SquareP (λ i j → isOfHLevelSuc 1 (isprop _ _))
(isProp→PathP (λ i₁ → isprop north (merid y i₁)) Bnorth
(subst (B north) (merid a) Bnorth))
(isProp→PathP (λ i₁ → isprop south (merid y i₁))
(subst (λ x₁ → B x₁ north) (merid a) Bnorth)
(subst (λ x₁ → B x₁ x₁) (merid a) Bnorth))
(isProp→PathP (λ i₁ → isprop (merid x i₁) north) Bnorth
(subst (λ x₁ → B x₁ north) (merid a) Bnorth))
(isProp→PathP (λ i₁ → isprop (merid x i₁) south)
(subst (B north) (merid a) Bnorth)
(subst (λ x₁ → B x₁ x₁) (merid a) Bnorth)) i j
{- Clever proof:
suspToPropElim2 a isProp Bnorth =
suspToPropElim a (λ x → isOfHLevelΠ 1 λ y → isProp x y)
(suspToPropElim a (λ x → isProp north x) Bnorth)
-}
funSpaceSuspIso : ∀ {ℓ ℓ'} {A : Type ℓ} {B : Type ℓ'}
→ Iso (Σ[ x ∈ B ] Σ[ y ∈ B ] (A → x ≡ y)) (Susp A → B)
Iso.fun funSpaceSuspIso (x , y , f) north = x
Iso.fun funSpaceSuspIso (x , y , f) south = y
Iso.fun funSpaceSuspIso (x , y , f) (merid a i) = f a i
Iso.inv funSpaceSuspIso f = (f north) , (f south , (λ x → cong f (merid x)))
Iso.rightInv funSpaceSuspIso f = funExt λ {north → refl
; south → refl
; (merid a i) → refl}
Iso.leftInv funSpaceSuspIso _ = refl
toSusp : (A : Pointed ℓ) → typ A → typ (Ω (Susp∙ (typ A)))
toSusp A x = merid x ∙ merid (pt A) ⁻¹
toSuspPointed : (A : Pointed ℓ) → A →∙ Ω (Susp∙ (typ A))
fst (toSuspPointed A) = toSusp A
snd (toSuspPointed A) = rCancel (merid (pt A))
module _ {ℓ ℓ' : Level} {A : Pointed ℓ} {B : Pointed ℓ'} where
fromSusp→toΩ : Susp∙ (typ A) →∙ B → (A →∙ Ω B)
fst (fromSusp→toΩ f) x = sym (snd f) ∙∙ cong (fst f) (toSusp A x) ∙∙ snd f
snd (fromSusp→toΩ f) =
cong (sym (snd f) ∙∙_∙∙ (snd f))
(cong (cong (fst f))
(rCancel (merid (pt A))))
∙ ∙∙lCancel (snd f)
toΩ→fromSusp : A →∙ Ω B → Susp∙ (typ A) →∙ B
fst (toΩ→fromSusp f) north = pt B
fst (toΩ→fromSusp f) south = pt B
fst (toΩ→fromSusp f) (merid a i) = fst f a i
snd (toΩ→fromSusp f) = refl
ΩSuspAdjointIso : Iso (A →∙ Ω B) (Susp∙ (typ A) →∙ B)
fun ΩSuspAdjointIso = toΩ→fromSusp
inv ΩSuspAdjointIso = fromSusp→toΩ
rightInv ΩSuspAdjointIso f =
ΣPathP (funExt
(λ { north → sym (snd f)
; south → sym (snd f) ∙ cong (fst f) (merid (pt A))
; (merid a i) j →
hcomp (λ k → λ { (i = i0) → snd f (~ j ∧ k)
; (i = i1) → compPath-filler'
(sym (snd f))
(cong (fst f) (merid (pt A))) k j
; (j = i1) → fst f (merid a i)})
(fst f (compPath-filler (merid a) (sym (merid (pt A))) (~ j) i))})
, λ i j → snd f (~ i ∨ j))
leftInv ΩSuspAdjointIso f =
→∙Homogeneous≡ (isHomogeneousPath _ _)
(funExt λ x → sym (rUnit _)
∙ cong-∙ (fst (toΩ→fromSusp f)) (merid x) (sym (merid (pt A)))
∙ cong (fst f x ∙_) (cong sym (snd f))
∙ sym (rUnit _))
IsoΩFunSuspFun : Iso (typ (Ω (A →∙ B ∙))) (Susp∙ (typ A) →∙ B)
IsoΩFunSuspFun = compIso (ΩfunExtIso A B) ΩSuspAdjointIso
| {
"alphanum_fraction": 0.5773102736,
"avg_line_length": 43.7740112994,
"ext": "agda",
"hexsha": "2315c9106f2b405056dca3615b0e628628c78ace",
"lang": "Agda",
"max_forks_count": null,
"max_forks_repo_forks_event_max_datetime": null,
"max_forks_repo_forks_event_min_datetime": null,
"max_forks_repo_head_hexsha": "b1d105aeeab1ba9888394c6a919b99a476390b7b",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "ecavallo/cubical",
"max_forks_repo_path": "Cubical/HITs/Susp/Properties.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "b1d105aeeab1ba9888394c6a919b99a476390b7b",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "ecavallo/cubical",
"max_issues_repo_path": "Cubical/HITs/Susp/Properties.agda",
"max_line_length": 89,
"max_stars_count": null,
"max_stars_repo_head_hexsha": "b1d105aeeab1ba9888394c6a919b99a476390b7b",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "ecavallo/cubical",
"max_stars_repo_path": "Cubical/HITs/Susp/Properties.agda",
"max_stars_repo_stars_event_max_datetime": null,
"max_stars_repo_stars_event_min_datetime": null,
"num_tokens": 2907,
"size": 7748
} |
------------------------------------------------------------------------------
-- Testing a non-admissible property from the HALO paper
------------------------------------------------------------------------------
{-# OPTIONS --exact-split #-}
{-# OPTIONS --no-sized-types #-}
{-# OPTIONS --no-universe-polymorphism #-}
{-# OPTIONS --without-K #-}
module FOT.FOTC.UnguardedCorecursion.HALO where
-- open import Common.FOL.Relation.Binary.EqReasoning
-- open import FOTC.Base
-- open import FOTC.Base.List
-- open import FOTC.Base.List.PropertiesI
-- open import FOTC.Data.Conat
-- open import FOTC.Data.Conat.PropertiesI
-- open import FOTC.Data.Nat
-- open import FOTC.Data.Stream.Type
-- open import FOTC.Data.Stream.Equality.PropertiesI
-- open import FOTC.Relation.Binary.Bisimilarity.PropertiesI
-- open import FOTC.Relation.Binary.Bisimilarity.Type
-- ------------------------------------------------------------------------------
-- -- The HALO paper states the property
-- --
-- -- ∀ x . f x ≠ ones (1)
-- --
-- -- cannot be proved because it is a non-admissible one.
-- postulate
-- ones : D
-- ones-eq : ones ≡ succ₁ zero ∷ ones
-- postulate
-- f : D → D
-- f-eq₁ : ∀ n → f (succ₁ n) ≡ succ₁ zero ∷ f n
-- f-eq₂ : f zero ≡ zero ∷ []
-- ------------------------------------------------------------------------------
-- -- Auxiliary properties
-- fCong : ∀ {m n} → m ≡ n → f m ≡ f n
-- fCong refl = refl
-- succ-∞-Conat : Conat (succ₁ ∞)
-- succ-∞-Conat = subst Conat ∞-eq ∞-Conat
-- ones-Stream : Stream ones
-- ones-Stream = Stream-coind A h refl
-- where
-- A : D → Set
-- A xs = xs ≡ xs
-- h : A ones → ∃[ x' ] ∃[ xs' ] ones ≡ x' ∷ xs' ∧ A xs'
-- h _ = succ₁ zero , ones , ones-eq , refl
-- f-∞-Stream : Stream (f ∞)
-- f-∞-Stream = Stream-coind A h refl
-- where
-- A : D → Set
-- A xs = f xs ≡ f xs
-- h : A (f ∞) → ∃[ x' ] ∃[ xs' ] f ∞ ≡ x' ∷ xs' ∧ A xs'
-- h Af∞ = succ₁ zero , f ∞ , trans (fCong ∞-eq) (f-eq₁ ∞) , Af∞
-- ------------------------------------------------------------------------------
-- -- A proof of (1) adding the N totality hypothesis.
-- thm₁ : ∀ {n} → N n → f n ≢ ones
-- thm₁ nzero h = 0≢S (∧-proj₁ (∷-injective helper))
-- where
-- helper : zero ∷ [] ≡ succ₁ zero ∷ ones
-- helper = trans₂ (sym f-eq₂) h ones-eq
-- thm₁ (nsucc {n} Nn) h = thm₁ Nn (∧-proj₂ (∷-injective helper))
-- where
-- helper : succ₁ zero ∷ f n ≡ succ₁ zero ∷ ones
-- helper = trans₂ (sym (f-eq₁ n)) h ones-eq
-- ------------------------------------------------------------------------------
-- -- A proof of (1) adding the N totality hypothesis and replacing the
-- -- propositional equality by the bisimilarity relation.
-- thm₂ : ∀ {n} → N n → f n ≉ ones
-- thm₂ nzero h with ≈-out h
-- ... | x' , xs' , ys' , prf₁ , prf₂ , prf₃ = 0≢S (trans (sym x'≡0) x'≡1)
-- where
-- x'≡0 : x' ≡ zero
-- x'≡0 = ∧-proj₁ (∷-injective (trans (sym prf₁) f-eq₂))
-- x'≡1 : x' ≡ succ₁ zero
-- x'≡1 = ∧-proj₁ (∷-injective (trans (sym prf₂) ones-eq))
-- thm₂ (nsucc {n} Nn) h with ≈-out h
-- ... | x' , xs' , ys' , prf₁ , prf₂ , prf₃ = thm₂ Nn (∷-injective≈ helper)
-- where
-- xs'≡fn : xs' ≡ f n
-- xs'≡fn = ∧-proj₂ (∷-injective (trans (sym prf₁) (f-eq₁ n)))
-- ys'≡ones : ys' ≡ ones
-- ys'≡ones = ∧-proj₂ (∷-injective (trans (sym prf₂) ones-eq))
-- helper : x' ∷ f n ≈ x' ∷ ones
-- helper = ≈-in ( x'
-- , xs'
-- , ys'
-- , ∷-rightCong (sym xs'≡fn)
-- , ∷-rightCong (sym ys'≡ones)
-- , prf₃
-- )
-- ------------------------------------------------------------------------------
-- -- A proof of the negation of (1) adding the Conat totality hypothesis
-- -- and replacing the propositional equality by the bisimilarity
-- -- relation.
-- thm₃ : ∃[ n ] (Conat n ∧ f n ≈ ones)
-- thm₃ = ∞ , ∞-Conat , ≈-coind B h (refl , refl)
-- where
-- B : D → D → Set
-- B xs ys = xs ≡ xs ∧ ys ≡ ys
-- h : B (f ∞) ones →
-- ∃[ x' ] ∃[ xs' ] ∃[ ys' ] f ∞ ≡ x' ∷ xs' ∧ ones ≡ x' ∷ ys' ∧ B xs' ys'
-- h Bh' = succ₁ zero , f ∞ , ones , trans (fCong ∞-eq) (f-eq₁ ∞) , ones-eq , Bh'
------------------------------------------------------------------------------
-- References
--
-- Vytiniotis, D., Peyton Jones, S., Rosén, D. and Claessen,
-- K. (2013). HALO: Haskell to Logic thorugh Denotational
-- Semantics. In: Proceedings of the 40th annual ACM SIGPLAN-SIGACT
-- symposium on Principles of programming languages (POPL’13),
-- pp. 431–442.
| {
"alphanum_fraction": 0.4705753664,
"avg_line_length": 33.3649635036,
"ext": "agda",
"hexsha": "836b3de30a6d5b1b47f129c774c6b4863c8cc286",
"lang": "Agda",
"max_forks_count": 3,
"max_forks_repo_forks_event_max_datetime": "2018-03-14T08:50:00.000Z",
"max_forks_repo_forks_event_min_datetime": "2016-09-19T14:18:30.000Z",
"max_forks_repo_head_hexsha": "2fc9f2b81052a2e0822669f02036c5750371b72d",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "asr/fotc",
"max_forks_repo_path": "notes/FOT/FOTC/UnguardedCorecursion/HALO.agda",
"max_issues_count": 2,
"max_issues_repo_head_hexsha": "2fc9f2b81052a2e0822669f02036c5750371b72d",
"max_issues_repo_issues_event_max_datetime": "2017-01-01T14:34:26.000Z",
"max_issues_repo_issues_event_min_datetime": "2016-10-12T17:28:16.000Z",
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "asr/fotc",
"max_issues_repo_path": "notes/FOT/FOTC/UnguardedCorecursion/HALO.agda",
"max_line_length": 83,
"max_stars_count": 11,
"max_stars_repo_head_hexsha": "2fc9f2b81052a2e0822669f02036c5750371b72d",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "asr/fotc",
"max_stars_repo_path": "notes/FOT/FOTC/UnguardedCorecursion/HALO.agda",
"max_stars_repo_stars_event_max_datetime": "2021-09-12T16:09:54.000Z",
"max_stars_repo_stars_event_min_datetime": "2015-09-03T20:53:42.000Z",
"num_tokens": 1544,
"size": 4571
} |
-- Andreas, 2011-09-13, shrunk from Data.Colist
-- {-# OPTIONS -v tc.lhs.unify:15 #-}
{-# OPTIONS --universe-polymorphism #-}
module TransColist where
open import Common.Level
open import Common.Coinduction
-- From Relation.Binary.Core:
------------------------------------------------------------------------
-- Binary relations
-- Heterogeneous binary relations
REL : ∀ {a b} → Set a → Set b → (ℓ : Level) → Set (a ⊔ b ⊔ lsuc ℓ)
REL A B ℓ = A → B → Set ℓ
-- Homogeneous binary relations
Rel : ∀ {a} → Set a → (ℓ : Level) → Set (a ⊔ lsuc ℓ)
Rel A ℓ = REL A A ℓ
-- Generalised transitivity.
Trans : ∀ {a b c ℓ₁ ℓ₂ ℓ₃} {A : Set a} {B : Set b} {C : Set c} →
REL A B ℓ₁ → REL B C ℓ₂ → REL A C ℓ₃ → Set _
Trans P Q R = ∀ {i j k} → P i j → Q j k → R i k
Transitive : ∀ {a ℓ} {A : Set a} → Rel A ℓ → Set _
Transitive _∼_ = Trans _∼_ _∼_ _∼_
infixr 5 _∷_
data Colist {a} (A : Set a) : Set a where
[] : Colist A
_∷_ : (x : A) (xs : ∞ (Colist A)) → Colist A
infix 4 _≈_
data _≈_ {a} {A : Set a} : (xs ys : Colist A) → Set a where
[] : [] ≈ []
_∷_ : ∀ x {xs ys} (xs≈ : ∞ (♭ xs ≈ ♭ ys)) → x ∷ xs ≈ x ∷ ys
postulate
a : Level
A : Set a
{- succeeds:
trans : -- forall {a}{A : Set a}
forall {xs ys zs : Colist A} →
xs ≈ ys → ys ≈ zs → xs ≈ zs
-}
-- succeeds:
-- trans : forall {a}{A : Set a}{xs ys zs : Colist A} → xs ≈ ys → ys ≈ zs → xs ≈ zs
trans : Transitive (_≈_ {A = A})
trans [] [] = []
trans (x ∷ xs≈) (.x ∷ ys≈) = x ∷ ♯ trans (♭ xs≈) (♭ ys≈)
| {
"alphanum_fraction": 0.4883570505,
"avg_line_length": 24.935483871,
"ext": "agda",
"hexsha": "ac7516b7d0f070e0a51b9fcc5a15deffa4d3774e",
"lang": "Agda",
"max_forks_count": 1,
"max_forks_repo_forks_event_max_datetime": "2019-03-05T20:02:38.000Z",
"max_forks_repo_forks_event_min_datetime": "2019-03-05T20:02:38.000Z",
"max_forks_repo_head_hexsha": "6043e77e4a72518711f5f808fb4eb593cbf0bb7c",
"max_forks_repo_licenses": [
"BSD-3-Clause"
],
"max_forks_repo_name": "alhassy/agda",
"max_forks_repo_path": "test/Succeed/TransColist.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "6043e77e4a72518711f5f808fb4eb593cbf0bb7c",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"BSD-3-Clause"
],
"max_issues_repo_name": "alhassy/agda",
"max_issues_repo_path": "test/Succeed/TransColist.agda",
"max_line_length": 84,
"max_stars_count": 3,
"max_stars_repo_head_hexsha": "6043e77e4a72518711f5f808fb4eb593cbf0bb7c",
"max_stars_repo_licenses": [
"BSD-3-Clause"
],
"max_stars_repo_name": "alhassy/agda",
"max_stars_repo_path": "test/Succeed/TransColist.agda",
"max_stars_repo_stars_event_max_datetime": "2015-12-07T20:14:00.000Z",
"max_stars_repo_stars_event_min_datetime": "2015-03-28T14:51:03.000Z",
"num_tokens": 612,
"size": 1546
} |
import Parametric.Syntax.Type as Type
module Parametric.Syntax.MType where
module Structure (Base : Type.Structure) where
open Type.Structure Base
mutual
-- Derived from CBPV
data ValType : Set where
U : (c : CompType) → ValType
B : (ι : Base) → ValType
vUnit : ValType
_v×_ : (τ₁ : ValType) → (τ₂ : ValType) → ValType
_v+_ : (τ₁ : ValType) → (τ₂ : ValType) → ValType
-- Same associativity as the standard _×_
infixr 2 _v×_
data CompType : Set where
F : ValType → CompType
_⇛_ : ValType → CompType → CompType
-- We did not use this in CBPV, so dropped.
-- _Π_ : CompType → CompType → CompType
cbnToCompType : Type → CompType
cbnToCompType (base ι) = F (B ι)
cbnToCompType (σ ⇒ τ) = U (cbnToCompType σ) ⇛ cbnToCompType τ
cbvToValType : Type → ValType
cbvToValType (base ι) = B ι
cbvToValType (σ ⇒ τ) = U (cbvToValType σ ⇛ F (cbvToValType τ))
open import Base.Syntax.Context ValType public
using ()
renaming
( ∅ to ∅∅
; _•_ to _••_
; mapContext to mapValCtx
; Var to ValVar
; Context to ValContext
; this to vThis; that to vThat
; _≼_ to _≼≼_
; weaken-var to weaken-val-var
; keep_•_ to keep_••_
; drop_•_ to drop_••_
; ≼-refl to ≼≼-refl
; ≼-trans to ≼≼-trans)
cbnToValType : Type → ValType
cbnToValType τ = U (cbnToCompType τ)
cbvToCompType : Type → CompType
cbvToCompType τ = F (cbvToValType τ)
fromCBNCtx : Context → ValContext
fromCBNCtx Γ = mapValCtx cbnToValType Γ
fromCBVCtx : Context → ValContext
fromCBVCtx Γ = mapValCtx cbvToValType Γ
open import Data.List
open Data.List using (List) public
fromCBVToCompList : Context → List CompType
fromCBVToCompList Γ = mapValCtx cbvToCompType Γ
fromVar : ∀ {Γ τ} → (f : Type → ValType) → Var Γ τ → ValVar (mapValCtx f Γ) (f τ)
fromVar {x • Γ} f this = vThis
fromVar {x • Γ} f (that v) = vThat (fromVar f v)
| {
"alphanum_fraction": 0.632166413,
"avg_line_length": 28.1571428571,
"ext": "agda",
"hexsha": "a8a2ff40531b9d5178f001391047709afacf90ff",
"lang": "Agda",
"max_forks_count": 1,
"max_forks_repo_forks_event_max_datetime": "2016-02-18T12:26:44.000Z",
"max_forks_repo_forks_event_min_datetime": "2016-02-18T12:26:44.000Z",
"max_forks_repo_head_hexsha": "39bb081c6f192bdb87bd58b4a89291686d2d7d03",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "inc-lc/ilc-agda",
"max_forks_repo_path": "Parametric/Syntax/MType.agda",
"max_issues_count": 6,
"max_issues_repo_head_hexsha": "39bb081c6f192bdb87bd58b4a89291686d2d7d03",
"max_issues_repo_issues_event_max_datetime": "2017-05-04T13:53:59.000Z",
"max_issues_repo_issues_event_min_datetime": "2015-07-01T18:09:31.000Z",
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "inc-lc/ilc-agda",
"max_issues_repo_path": "Parametric/Syntax/MType.agda",
"max_line_length": 83,
"max_stars_count": 10,
"max_stars_repo_head_hexsha": "39bb081c6f192bdb87bd58b4a89291686d2d7d03",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "inc-lc/ilc-agda",
"max_stars_repo_path": "Parametric/Syntax/MType.agda",
"max_stars_repo_stars_event_max_datetime": "2019-07-19T07:06:59.000Z",
"max_stars_repo_stars_event_min_datetime": "2015-03-04T06:09:20.000Z",
"num_tokens": 719,
"size": 1971
} |
module Delay where
open import OscarPrelude
mutual
data Delay (i : Size) (A : Set) : Set where
now : A → Delay i A
later : ∞Delay i A → Delay i A
record ∞Delay (i : Size) (A : Set) : Set where
coinductive
field
force : {j : Size< i} → Delay j A
open ∞Delay public
private
module BindDelay
where
mutual
bindDelay : ∀ {i A B} → Delay i A → (A → Delay i B) → Delay i B
bindDelay (now a) f = f a
bindDelay (later ∞a) f = later (bind∞Delay ∞a f)
bind∞Delay : ∀ {i A B} → ∞Delay i A → (A → Delay i B) → ∞Delay i B
force (bind∞Delay ∞a f) = bindDelay (force ∞a) f
module _
where
open BindDelay
open BindDelay public using () renaming (bind∞Delay to _∞>>=_)
instance FunctorDelay : {i : Size} → Functor (Delay i)
Functor.fmap FunctorDelay f x = bindDelay x $ now ∘ f
instance ApplicativeDelay : {i : Size} → Applicative (Delay i)
Applicative.pure ApplicativeDelay x = now x
Applicative._<*>_ ApplicativeDelay (now f) x = f <$> x
Applicative._<*>_ ApplicativeDelay (later ∞f) x = later ∘ bind∞Delay ∞f $ flip fmap x
Applicative.super ApplicativeDelay = FunctorDelay
instance MonadDelay : {i : Size} → Monad (Delay i)
Monad._>>=_ MonadDelay = bindDelay
Monad.super MonadDelay = ApplicativeDelay
{-# DISPLAY BindDelay.bindDelay x f = x >>= f #-}
mutual
data _∼_ {i : Size} {A : Set} : (a? b? : Delay ∞ A) → Set where
∼now : ∀ a → now a ∼ now a
∼later : ∀ {a∞ b∞} (eq : a∞ ∞∼⟨ i ⟩∼ b∞) → later a∞ ∼ later b∞
_∼⟨_⟩∼_ = λ {A} a? i b? → _∼_ {i}{A} a? b?
record _∞∼⟨_⟩∼_ {A} (a∞ : ∞Delay ∞ A) i (b∞ : ∞Delay ∞ A) : Set where
coinductive
field
∼force : {j : Size< i} → force a∞ ∼⟨ j ⟩∼ force b∞
open _∞∼⟨_⟩∼_ public
_∞∼_ = λ {i} {A} a∞ b∞ → _∞∼⟨_⟩∼_ {A} a∞ i b∞
mutual
∼refl : ∀{i A} (a? : Delay ∞ A) → a? ∼⟨ i ⟩∼ a?
∼refl (now a) = ∼now a
∼refl (later a∞) = ∼later (∞∼refl a∞)
∞∼refl : ∀{i A} (a∞ : ∞Delay ∞ A) → a∞ ∞∼⟨ i ⟩∼ a∞
∼force (∞∼refl a∞) = ∼refl (force a∞)
mutual
∼sym : ∀{i A}{a? b? : Delay ∞ A } → a? ∼⟨ i ⟩∼ b? → b? ∼⟨ i ⟩∼ a?
∼sym (∼now a) = ∼now a
∼sym (∼later eq) = ∼later (∞∼sym eq)
∞∼sym : ∀{i A}{a∞ b∞ : ∞Delay ∞ A} → a∞ ∞∼⟨ i ⟩∼ b∞ → b∞ ∞∼⟨ i ⟩∼ a∞
∼force (∞∼sym eq) = ∼sym (∼force eq)
mutual
∼trans : ∀{i A}{a? b? c? : Delay ∞ A} →
a? ∼⟨ i ⟩∼ b? → b? ∼⟨ i ⟩∼ c? → a? ∼⟨ i ⟩∼ c?
∼trans (∼now a) (∼now .a) = ∼now a
∼trans (∼later eq) (∼later eq′) = ∼later (∞∼trans eq eq′)
∞∼trans : ∀{i A}{a∞ b∞ c∞ : ∞Delay ∞ A} →
a∞ ∞∼⟨ i ⟩∼ b∞ → b∞ ∞∼⟨ i ⟩∼ c∞ → a∞ ∞∼⟨ i ⟩∼ c∞
∼force (∞∼trans eq eq′) = ∼trans (∼force eq) (∼force eq′)
--∼setoid : (i : Size) (A : Set) → Setoid lzero lzero
--∞∼setoid : (i : Size) (A : Set) → Setoid lzero lzero
mutual
bind-assoc : ∀{i A B C} (m : Delay ∞ A)
{k : A → Delay ∞ B} {l : B → Delay ∞ C} →
((m >>= k) >>= l) ∼⟨ i ⟩∼ (m >>= λ a → (k a >>= l))
bind-assoc (now a) = ∼refl _
bind-assoc (later a∞) = ∼later (∞bind-assoc a∞)
∞bind-assoc : ∀{i A B C} (a∞ : ∞Delay ∞ A)
{k : A → Delay ∞ B} {l : B → Delay ∞ C} →
((a∞ ∞>>= k) ∞>>= l) ∞∼⟨ i ⟩∼ (a∞ ∞>>= λ a → (k a >>= l))
∼force (∞bind-assoc a∞) = bind-assoc (force a∞)
mutual
bind-cong-l : ∀{i A B}{a? b? : Delay ∞ A} → a? ∼⟨ i ⟩∼ b? →
(k : A → Delay ∞ B) → (a? >>= k) ∼⟨ i ⟩∼ (b? >>= k)
bind-cong-l (∼now a) k = ∼refl _
bind-cong-l (∼later eq) k = ∼later (∞bind-cong-l eq k)
∞bind-cong-l : ∀{i A B}{a∞ b∞ : ∞Delay ∞ A} → a∞ ∞∼⟨ i ⟩∼ b∞ →
(k : A → Delay ∞ B) → (a∞ ∞>>= k) ∞∼⟨ i ⟩∼ (b∞ ∞>>= k)
∼force (∞bind-cong-l eq k) = bind-cong-l (∼force eq) k
mutual
bind-cong-r : ∀{i A B}(a? : Delay ∞ A){k l : A → Delay ∞ B} →
(∀ a → (k a) ∼⟨ i ⟩∼ (l a)) → (a? >>= k) ∼⟨ i ⟩∼ (a? >>= l)
bind-cong-r (now a) h = h a
bind-cong-r (later a∞) h = ∼later (∞bind-cong-r a∞ h)
∞bind-cong-r : ∀{i A B}(a∞ : ∞Delay ∞ A){k l : A → Delay ∞ B} →
(∀ a → (k a) ∼⟨ i ⟩∼ (l a)) → (a∞ ∞>>= k) ∞∼⟨ i ⟩∼ (a∞ ∞>>= l)
∼force (∞bind-cong-r a∞ h) = bind-cong-r (force a∞) h
map-compose : ∀{i A B C} (a? : Delay ∞ A) {f : A → B} {g : B → C} →
(g <$> (f <$> a?)) ∼⟨ i ⟩∼ ((g ∘ f) <$> a?)
map-compose a? = bind-assoc a?
map-cong : ∀{i A B}{a? b? : Delay ∞ A} (f : A → B) →
a? ∼⟨ i ⟩∼ b? → (f <$> a?) ∼⟨ i ⟩∼ (f <$> b?)
map-cong f eq = bind-cong-l eq (now ∘ f)
data _⇓_ {A : Set} : (a? : Delay ∞ A) (a : A) → Set where
now⇓ : ∀{a} → now a ⇓ a
later⇓ : ∀{a} {a∞ : ∞Delay ∞ A} → force a∞ ⇓ a → later a∞ ⇓ a
_⇓ : {A : Set} (x : Delay ∞ A) → Set
x ⇓ = ∃ λ a → x ⇓ a
map⇓ : ∀{A B}{a : A}{a? : Delay ∞ A}(f : A → B) → a? ⇓ a → (f <$> a?) ⇓ f a
map⇓ f now⇓ = now⇓
map⇓ f (later⇓ a⇓) = later⇓ (map⇓ f a⇓)
bind⇓ : ∀{A B}(f : A → Delay ∞ B){?a : Delay ∞ A}{a : A}{b : B} →
?a ⇓ a → f a ⇓ b → (?a >>= f) ⇓ b
bind⇓ f now⇓ q = q
bind⇓ f (later⇓ p) q = later⇓ (bind⇓ f p q)
infixl 4 _>>=⇓_
_>>=⇓_ : ∀{A B}{f : A → Delay ∞ B}{?a : Delay ∞ A}{a : A}{b : B} →
?a ⇓ a → f a ⇓ b → (?a >>= f) ⇓ b
_>>=⇓_ = bind⇓ _
infixl 4 _⇓>>=⇓_
_⇓>>=⇓_ : ∀{A B}{f : A → Delay ∞ B}{?a : Delay ∞ A}{b : B} →
(?a⇓ : ?a ⇓) → f (fst ?a⇓) ⇓ b → (?a >>= f) ⇓ b
_⇓>>=⇓_ (_ , a⇓) = bind⇓ _ a⇓
_⇓Dec>>=⇓_else⇓_ : ∀{A B}{f-yes : A → Delay ∞ B}{f-no : ¬ A → Delay ∞ B}{?a : Delay ∞ (Dec A)}{b : B} →
(?a⇓ : ?a ⇓) →
((a : A) → f-yes a ⇓ b) →
((¬a : ¬ A) → f-no ¬a ⇓ b) →
((?a >>= (λ { (yes y) → f-yes y ; (no n) → f-no n }))) ⇓ b
(yes y , y⇓) ⇓Dec>>=⇓ fy⇓ else⇓ fn⇓ = y⇓ >>=⇓ fy⇓ y
(no n , n⇓) ⇓Dec>>=⇓ fy⇓ else⇓ fn⇓ = n⇓ >>=⇓ fn⇓ n
_⇓DecEq>>=⇓_else⇓_ : ∀{A : Set} {A₁ A₂ : A} {B}{f-yes : A₁ ≡ A₂ → Delay ∞ B}{f-no : A₁ ≢ A₂ → Delay ∞ B}{?a : Delay ∞ (Dec (A₁ ≡ A₂))}{b : B} →
(?a⇓ : ?a ⇓) →
((eq : A₁ ≡ A₂) → f-yes eq ⇓ b) →
((¬eq : A₁ ≢ A₂) → f-no ¬eq ⇓ b) →
((?a >>= (λ { (yes refl) → f-yes refl ; (no n) → f-no n }))) ⇓ b
(yes refl , y⇓) ⇓DecEq>>=⇓ fy⇓ else⇓ fn⇓ = y⇓ >>=⇓ fy⇓ refl
(no n , n⇓) ⇓DecEq>>=⇓ fy⇓ else⇓ fn⇓ = n⇓ >>=⇓ fn⇓ n
app⇓ : ∀{A}{B}{f? : Delay ∞ (A → B)}{f : A → B}{x? : Delay ∞ A}{x : A} → f? ⇓ f → x? ⇓ x → (f? <*> x?) ⇓ f x
app⇓ now⇓ now⇓ = now⇓
app⇓ now⇓ (later⇓ x?) = later⇓ $ map⇓ _ x?
app⇓ (later⇓ f?) now⇓ = later⇓ $ bind⇓ _ f? now⇓
app⇓ (later⇓ ⇓f) (later⇓ ⇓x) = later⇓ $ bind⇓ _ ⇓f $ later⇓ $ bind⇓ _ ⇓x now⇓
subst∼⇓ : ∀{A}{a? a?′ : Delay ∞ A}{a : A} → a? ⇓ a → a? ∼ a?′ → a?′ ⇓ a
subst∼⇓ now⇓ (∼now a) = now⇓
subst∼⇓ (later⇓ p) (∼later eq) = later⇓ (subst∼⇓ p (∼force eq))
traverse-list⇓ : ∀{A}{B} (f? : A → Delay ∞ B) → (∀ x → f? x ⇓) → (xs : List A) → traverse f? xs ⇓
traverse-list⇓ f? f?⇓ [] = [] , now⇓
traverse-list⇓ f? f?⇓ (x ∷ xs)
with f?⇓ x | traverse-list⇓ f? f?⇓ xs
… | y , y⇓ | ys , ys⇓ = y ∷ ys , app⇓ (map⇓ _ y⇓) ys⇓
| {
"alphanum_fraction": 0.4103241965,
"avg_line_length": 35.4039408867,
"ext": "agda",
"hexsha": "9e5b8325dd18a9107e73692c54d087929926ab76",
"lang": "Agda",
"max_forks_count": null,
"max_forks_repo_forks_event_max_datetime": null,
"max_forks_repo_forks_event_min_datetime": null,
"max_forks_repo_head_hexsha": "52e1cdbdee54d9a8eaee04ee518a0d7f61d25afb",
"max_forks_repo_licenses": [
"RSA-MD"
],
"max_forks_repo_name": "m0davis/oscar",
"max_forks_repo_path": "archive/agda-1/Delay.agda",
"max_issues_count": 1,
"max_issues_repo_head_hexsha": "52e1cdbdee54d9a8eaee04ee518a0d7f61d25afb",
"max_issues_repo_issues_event_max_datetime": "2019-05-11T23:33:04.000Z",
"max_issues_repo_issues_event_min_datetime": "2019-04-29T00:35:04.000Z",
"max_issues_repo_licenses": [
"RSA-MD"
],
"max_issues_repo_name": "m0davis/oscar",
"max_issues_repo_path": "archive/agda-1/Delay.agda",
"max_line_length": 143,
"max_stars_count": null,
"max_stars_repo_head_hexsha": "52e1cdbdee54d9a8eaee04ee518a0d7f61d25afb",
"max_stars_repo_licenses": [
"RSA-MD"
],
"max_stars_repo_name": "m0davis/oscar",
"max_stars_repo_path": "archive/agda-1/Delay.agda",
"max_stars_repo_stars_event_max_datetime": null,
"max_stars_repo_stars_event_min_datetime": null,
"num_tokens": 3752,
"size": 7187
} |
{-# OPTIONS --without-K #-}
{- This module serves to develop some basic theory about pointed types.
After defining the usual notions of pointed types, pointed equivalences,
and loop spaces, we derive a version of univalence for pointed equivalences
and observe that univalence between identical types is a pointed equivalence.
We define pointed versions of dependent sums and products using the usual
notion of pointed families and observe that they commute in a certain sense
with taking loop spaces.
We finish by deriving a generalization to n-truncation and n-th loop spaces
of the fact allowing us to 'forget' contractible components in a dependent
sum type that will be needed in the Hierarchy module. -}
module Universe.Utility.Pointed where
open import lib.Basics
open import lib.NType2
open import lib.types.Nat hiding (_+_)
open import lib.types.Pi
open import lib.types.Sigma
open import lib.types.TLevel
open import Universe.Utility.General
open import Universe.Utility.TruncUniverse
{- Pointed types.
A pointed type is a type (base) together with a chosen element (pt).
The loop space construction Ω takes a pointed type and returns the type
of all loops at the given basepoint. The trivial loop is taken as
canonical element, thus forming a new pointed type. -}
Type• : (i : ULevel) → Type (lsucc i)
Type• i = Σ (Type i) (idf _)
module _ {i} (X : Type• i) where
base = fst X
pt = snd X
-- Alternate definition: Σ (n -Type i) ⟦_⟧
_-Type•_ : (n : ℕ₋₂) (i : ULevel) → Type (lsucc i)
n -Type• i = Σ (Type• i) (has-level n ∘ base)
-- For alternate definition: Σ-≤ (n -Type-≤ i) raise
_-Type•-≤_ : (n : ℕ₋₂) (i : ULevel) → S n -Type lsucc i
n -Type•-≤ i = (n -Type• i
, equiv-preserves-level Σ-comm-snd
(snd (Σ-≤ (n -Type-≤ i) raise)))
{- Pointed equivalences.
An equivalence of pointed types is an equivalences of the bases
that preserves the points -}
_≃•_ : ∀ {i j} → Type• i → Type• j → Set (i ⊔ j)
A ≃• B = Σ (base A ≃ base B) (λ f → –> f (pt A) == pt B)
ide• : ∀ {i} (X : Type• i) → X ≃• X
ide• _ = ide _ , idp
_∘e•_ : ∀ {i j k} {X : Type• i} {Y : Type• j} {Z : Type• k}
→ Y ≃• Z → X ≃• Y → X ≃• Z
(u , p) ∘e• (v , q) = (u ∘e v , ap (–> u) q ∙ p)
_⁻¹• : ∀ {i j} {X : Type• i} {Y : Type• j} → X ≃• Y → Y ≃• X
(u , p) ⁻¹• = (u ⁻¹ , ap (<– u) (! p) ∙ <–-inv-l u _)
-- Equational reasoning for pointed equivalences.
infix 2 _≃•∎
infixr 2 _≃•⟨_⟩_
_≃•⟨_⟩_ : ∀ {i j k} (X : Type• i) {Y : Type• j} {Z : Type• k}
→ X ≃• Y → Y ≃• Z → X ≃• Z
_ ≃•⟨ u ⟩ v = v ∘e• u
_≃•∎ : ∀ {i} (X : Type• i) → X ≃• X
_≃•∎ = ide•
-- The loop space construction.
Ω : ∀ {i} → Type• i → Type• i
Ω (A , a) = (a == a , idp)
Ω-≤ : ∀ {i} {n : ℕ₋₂} → (S n) -Type• i → n -Type• i
Ω-≤ ((A , a) , t) = (Ω (A , a) , t a a)
-- Loop spaces are preserved by pointed equivalences.
equiv-Ω : ∀ {i j} {X : Type• i} {Y : Type• j} → X ≃• Y → Ω X ≃• Ω Y
equiv-Ω (u , p) = split u p where
split : ∀ u {a} {b} → –> u a == b → Ω (_ , a) ≃• Ω (_ , b)
split u idp = (equiv-ap u _ _ , idp)
equiv-Ω^ : ∀ {i j} {X : Type• i} {Y : Type• j} (n : ℕ)
→ X ≃• Y → (Ω ^ n) X ≃• (Ω ^ n) Y
equiv-Ω^ 0 e = e
equiv-Ω^ (S n) e = equiv-Ω^ n (equiv-Ω e)
{- We call a pointed type n-truncated if its base is.
Constructing the loop space decrements the truncation level. -}
has-level• : ∀ {i} → ℕ₋₂ → Type• i → Type i
has-level• n = has-level n ∘ base
trunc-many : ∀ {i} {X : Type• i} {k : ℕ} (n : ℕ)
→ has-level• (k + n -2) X
→ has-level• (k -2) ((Ω ^ n) X)
trunc-many 0 t = t
trunc-many (S n) t = trunc-many n (t _ _)
--Ω^-≤ : ∀ {i} {k : ℕ} (n : ℕ) → (k + n -2) -Type• i → (k -2) -Type• i
--Ω^-≤ O X = X
--Ω^-≤ (S n) X = Ω^-≤ n (Ω-≤ X)
Ω^-≤ : ∀ {i} {k : ℕ} (n : ℕ) → (k + n -2) -Type• i → (k -2) -Type• i
Ω^-≤ n (X , t) = ((Ω ^ n) X , trunc-many n t)
Ω^-≤' : ∀ {i} {k : ℕ} (n : ℕ) → (n + k -2) -Type• i → (k -2) -Type• i
Ω^-≤' n (X , t) =
((Ω ^ n) X , trunc-many n (transport (λ z → has-level• (z -2) X)
(+-comm _ n) t))
{- Pointedness allows for a more direct notion of contractibility.
Beware that is-contr• will be equivalent --- not definitionally equal ---
to has-level∙ ⟨-2⟩. -}
module _ {i} (X : Type• i) where
is-contr• : Type i
is-contr• = ∀ a → pt X == a
{- Since pointed types are always inhabited,
being contractible and propositional is equivalent. -}
module _ {i} {X : Type• i} where
contr•-equiv-contr : is-contr• X ≃ is-contr (base X)
contr•-equiv-contr = prop-equiv'
(λ c → Π-level (λ a → raise-level-<T (ltSR ltS) c _ _))
(cst is-contr-is-prop)
(λ x → (pt X , x))
(λ y _ → prop-has-all-paths (contr-is-prop y) _ _)
is-contr•-is-prop : is-prop (is-contr• X)
is-contr•-is-prop = equiv-preserves-level (contr•-equiv-contr ⁻¹)
is-contr-is-prop
prop-equiv-contr : is-prop (base X) ≃ is-contr (base X)
prop-equiv-contr = prop-equiv is-prop-is-prop
is-contr-is-prop
(inhab-prop-is-contr (pt X))
contr-is-prop
contr•-equiv-prop : is-contr• X ≃ is-prop (base X)
contr•-equiv-prop = prop-equiv-contr ⁻¹ ∘e contr•-equiv-contr
-- ** Lemma 5.4 ***
{- The induction step for Lemma 7.2.9 in the HoTT Book is much
more complicated than neccesarry. Associating iterated loop spaces in
the reverse order, we can do away with the prerequisites 7.2.7 and 7.2.8
as well as further auxiliary steps. -}
has-level-equiv-contr-loops : ∀ {i} {n : ℕ} {A : Type i}
→ has-level (n -1) A
≃ ((a : A) → is-contr• ((Ω ^ n) (A , a)))
has-level-equiv-contr-loops {n = O} {A} =
is-prop A ≃⟨ prop-equiv-inhab-to-contr ⟩
(A → is-contr A) ≃⟨ equiv-Π-r (λ _ → contr•-equiv-contr ⁻¹) ⟩
((a : A) → is-contr• (A , a)) ≃∎
has-level-equiv-contr-loops {n = S n} {A} = equiv-Π-r lem where
lem = λ a →
(((b : A) → has-level ( n -1) (a == b)))
≃⟨ equiv-Π-r (λ _ → has-level-equiv-contr-loops) ⟩
(((b : A) (p : a == b) → is-contr• ((Ω ^ n) (a == b , p))))
≃⟨ Π₁-contr (pathfrom-is-contr _) ∘e curry-equiv ⁻¹ ⟩
is-contr• ((Ω ^ n) (a == a , idp))
≃∎
-- Pointed equivalences preserve (pointed) contractibility.
equiv-is-contr• : ∀ {i j} {X : Type• i} {Y : Type• j}
→ X ≃• Y → is-contr• X ≃ is-contr• Y
equiv-is-contr• (u , p) = contr•-equiv-contr ⁻¹
∘e equiv-level u
∘e contr•-equiv-contr
-- Univalence for pointed equivalences.
module _ {i} {A B : Type• i} where
ua•-equiv : (A ≃• B) ≃ (A == B)
ua•-equiv =
A ≃• B
≃⟨ ide _ ⟩
Σ (base A ≃ base B) (λ f → –> f (pt A) == pt B)
≃⟨ equiv-Σ-fst _ (snd (ua-equiv ⁻¹)) ⁻¹ ⟩
Σ (base A == base B) (λ q → coe q (pt A) == pt B)
≃⟨ equiv-Σ-snd (λ q → coe-equiv (ap (λ f → coe f (pt A) == pt B)
(! (ap-idf q)))) ⟩
Σ (base A == base B) (λ q → coe (ap (idf _) q) (pt A) == pt B)
≃⟨ equiv-Σ-snd (λ q → to-transp-equiv _ q ⁻¹) ⟩
Σ (base A == base B) (λ q → pt A == pt B [ idf _ ↓ q ])
≃⟨ =Σ-eqv _ _ ⟩
A == B
≃∎
ua• : A ≃• B → A == B
ua• = –> ua•-equiv
coe•-equiv : A == B → A ≃• B
coe•-equiv = <– ua•-equiv
-- Normal univalence can be made pointed in the endo-setting.
module _ {i} {A : Type i} where
ua-equiv• : (A ≃ A , ide _) ≃• (A == A , idp)
ua-equiv• = ((ua-equiv ⁻¹) , idp) ⁻¹•
-- *** Definition 4.1 ***
{- Pointed families.
A pointed family over a pointed type is a family over the base
together with a inhabitant of the family at the point.
Note that pointed types are equivalent to pointed families
over the pointed unit type (not shown here). -}
Fam• : ∀ {i} (X : Type• i) (j : ULevel) → Type (i ⊔ lsucc j)
Fam• X j = Σ (base X → Type j) (λ P → P (pt X))
-- We have fibered notions of the loop space contruction and n-truncatedness.
module _ {i} {X : Type• i} {j} where
-- *** Definition 4.3 ***
{- Note that the definition of the family of path types differs slightly from
that of the article, which would correspond to transport P p x == x.
We use dependent paths since this follows the design of the HoTT
community's Agda library. Clearly, both types are equivalent. -}
Ω̃ : Fam• X j → Fam• (Ω X) j
Ω̃ (P , x) = ((λ p → x == x [ P ↓ p ]) , idp)
fam-has-level : ℕ₋₂ → Fam• X j → Type (i ⊔ j)
fam-has-level n Q = (a : base X) → has-level n (fst Q a)
{- == Pointed dependent sums ==
Pointed families as defined above enable us to introduce a Σ-connective
for pointed types. Because of the abstract nature of some of our lemmata, we
give Σ• in its uncurried form and first define the type of its parameter. -}
Σ•-param : ∀ i j → Type (lsucc (i ⊔ j))
Σ•-param i j = Σ (Type• i) (λ X → Fam• X j)
module _ {i j} where
Ω-Σ•-param : Σ•-param i j → Σ•-param i j
Ω-Σ•-param (X , W) = (Ω X , Ω̃ W)
-- *** Definition 4.4 ***
Σ• : Σ•-param i j → Type• (i ⊔ j)
Σ• (X , Q) = (Σ (base X) (fst Q) , (pt X , snd Q))
-- *** Lemma 4.5 ***
{- Commutativity of pointed dependent sums and the loop space construction
will become an important technical tool, enabling us to work at a more
abstract level later on. -}
Ω-Σ•-comm : (R : Σ•-param i j) → Ω (Σ• R) ≃• Σ• (Ω-Σ•-param R)
Ω-Σ•-comm _ = (=Σ-eqv _ _ , idp) ⁻¹•
{- Pointed dependent products.
This is not quite the equivalent of Π for pointed types: the domain parameter
is just an ordinary non-pointed type. However, to enable our goal of
abstractly working with pointed types, defining this notion is useful. -}
Π•-param : ∀ i j → Type (lsucc (i ⊔ j))
Π•-param i j = Σ (Type i) (λ A → A → Type• j)
module _ {i j} where
Ω-Π•-param : Π•-param i j → Π•-param i j
Ω-Π•-param (A , F) = (A , Ω ∘ F)
-- *** Definition 4.6 ***
Π• : Π•-param i j → Type• (i ⊔ j)
Π• (A , Y) = (Π A (base ∘ Y) , pt ∘ Y)
-- *** Lemma 4.7 ***
{- Pointed dependent products and loop space construction on
its codomain parameter commute as well. -}
Ω-Π•-comm : (R : Π•-param i j) → Ω (Π• R) ≃• Π• (Ω-Π•-param R)
Ω-Π•-comm _ = (app=-equiv , idp)
Ω^-Π•-comm : (C : Type i) (F : C → Type• j) (n : ℕ)
→ (Ω ^ n) (Π• (C , F)) ≃• Π• (C , Ω ^ n ∘ F)
Ω^-Π•-comm C F 0 = ide• _
Ω^-Π•-comm C F (S n) = Ω^-Π•-comm C _ n ∘e• equiv-Ω^ n (Ω-Π•-comm _)
equiv-Π• : ∀ {i₀ i₁ j₀ j₁} {R₀ : Π•-param i₀ j₀} {R₁ : Π•-param i₁ j₁}
→ Σ (fst R₀ ≃ fst R₁) (λ u → ∀ a → snd R₀ (<– u a) ≃• snd R₁ a)
→ Π• R₀ ≃• Π• R₁
equiv-Π• (u , v) = (equiv-Π u (fst ∘ v) , λ= (snd ∘ v))
-- *** Lemma 5.1 ***
-- In an n-th loop space, we can forget components of truncation level n.
forget-Ω^-Σ•₂ : ∀ {i j} {X : Type• i} (Q : Fam• X j) (n : ℕ)
→ fam-has-level (n -2) Q → (Ω ^ n) (Σ• (X , Q)) ≃• (Ω ^ n) X
forget-Ω^-Σ•₂ {X = X} Q O h = (Σ₂-contr h , idp)
forget-Ω^-Σ•₂ {i} {X = X} Q (S n) h =
(Ω ^ (S n)) (Σ• (X , Q)) ≃•⟨ equiv-Ω^ n (Ω-Σ•-comm _) ⟩
(Ω ^ n) (Σ• (Ω X , Ω̃ Q)) ≃•⟨ forget-Ω^-Σ•₂ {i} _ n (λ _ → =-[-↓-]-level h) ⟩
(Ω ^ (S n)) X ≃•∎
| {
"alphanum_fraction": 0.5310296192,
"avg_line_length": 38.1952861953,
"ext": "agda",
"hexsha": "d351796aae7bc69d24ac21029e9619860841b70b",
"lang": "Agda",
"max_forks_count": null,
"max_forks_repo_forks_event_max_datetime": null,
"max_forks_repo_forks_event_min_datetime": null,
"max_forks_repo_head_hexsha": "c8fb8da3354fc9e0c430ac14160161759b4c5b37",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "sattlerc/HoTT-Agda",
"max_forks_repo_path": "Universe/Utility/Pointed.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "c8fb8da3354fc9e0c430ac14160161759b4c5b37",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "sattlerc/HoTT-Agda",
"max_issues_repo_path": "Universe/Utility/Pointed.agda",
"max_line_length": 80,
"max_stars_count": null,
"max_stars_repo_head_hexsha": "c8fb8da3354fc9e0c430ac14160161759b4c5b37",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "sattlerc/HoTT-Agda",
"max_stars_repo_path": "Universe/Utility/Pointed.agda",
"max_stars_repo_stars_event_max_datetime": null,
"max_stars_repo_stars_event_min_datetime": null,
"num_tokens": 4433,
"size": 11344
} |
------------------------------------------------------------------------
-- The Agda standard library
--
-- Fancy display functions for Vec-based tables
------------------------------------------------------------------------
{-# OPTIONS --safe --without-K #-}
module Text.Tabular.Vec where
open import Data.List.Base using (List)
open import Data.Product as Prod using (uncurry)
open import Data.String.Base using (String; rectangle; fromAlignment)
open import Data.Vec.Base
open import Function.Base
open import Text.Tabular.Base
display : ∀ {m n} → TabularConfig → Vec Alignment n → Vec (Vec String n) m →
List String
display c a = unsafeDisplay c
∘ toList
∘ map toList
∘ transpose
∘ map (uncurry rectangle ∘ unzip)
∘ transpose
∘ map (zip (map fromAlignment a))
| {
"alphanum_fraction": 0.5410798122,
"avg_line_length": 30.4285714286,
"ext": "agda",
"hexsha": "a9482eb019504a937819033f84ecd339d6e7e4f2",
"lang": "Agda",
"max_forks_count": 1,
"max_forks_repo_forks_event_max_datetime": "2021-11-04T06:54:45.000Z",
"max_forks_repo_forks_event_min_datetime": "2021-11-04T06:54:45.000Z",
"max_forks_repo_head_hexsha": "fb380f2e67dcb4a94f353dbaec91624fcb5b8933",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "DreamLinuxer/popl21-artifact",
"max_forks_repo_path": "agda-stdlib/src/Text/Tabular/Vec.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "fb380f2e67dcb4a94f353dbaec91624fcb5b8933",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "DreamLinuxer/popl21-artifact",
"max_issues_repo_path": "agda-stdlib/src/Text/Tabular/Vec.agda",
"max_line_length": 76,
"max_stars_count": 5,
"max_stars_repo_head_hexsha": "fb380f2e67dcb4a94f353dbaec91624fcb5b8933",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "DreamLinuxer/popl21-artifact",
"max_stars_repo_path": "agda-stdlib/src/Text/Tabular/Vec.agda",
"max_stars_repo_stars_event_max_datetime": "2020-10-10T21:41:32.000Z",
"max_stars_repo_stars_event_min_datetime": "2020-10-07T12:07:53.000Z",
"num_tokens": 174,
"size": 852
} |
open import Agda.Builtin.Equality
postulate
A : Set
mutual
F : ((@♭ _ : A) -> A) → A → A
F f = _
testF : {f : A -> A} → F f ≡ f
testF = refl
| {
"alphanum_fraction": 0.5,
"avg_line_length": 12.8333333333,
"ext": "agda",
"hexsha": "a9e16ca7b685ed38dcd83c28ae8c8e2023f9c38b",
"lang": "Agda",
"max_forks_count": 371,
"max_forks_repo_forks_event_max_datetime": "2022-03-30T19:00:30.000Z",
"max_forks_repo_forks_event_min_datetime": "2015-01-03T14:04:08.000Z",
"max_forks_repo_head_hexsha": "ed8ac6f4062ea8a20fa0f62d5db82d4e68278338",
"max_forks_repo_licenses": [
"BSD-3-Clause"
],
"max_forks_repo_name": "shlevy/agda",
"max_forks_repo_path": "test/Fail/Issue4390flat.agda",
"max_issues_count": 4066,
"max_issues_repo_head_hexsha": "ed8ac6f4062ea8a20fa0f62d5db82d4e68278338",
"max_issues_repo_issues_event_max_datetime": "2022-03-31T21:14:49.000Z",
"max_issues_repo_issues_event_min_datetime": "2015-01-10T11:24:51.000Z",
"max_issues_repo_licenses": [
"BSD-3-Clause"
],
"max_issues_repo_name": "shlevy/agda",
"max_issues_repo_path": "test/Fail/Issue4390flat.agda",
"max_line_length": 33,
"max_stars_count": 1989,
"max_stars_repo_head_hexsha": "ed8ac6f4062ea8a20fa0f62d5db82d4e68278338",
"max_stars_repo_licenses": [
"BSD-3-Clause"
],
"max_stars_repo_name": "shlevy/agda",
"max_stars_repo_path": "test/Fail/Issue4390flat.agda",
"max_stars_repo_stars_event_max_datetime": "2022-03-30T18:20:48.000Z",
"max_stars_repo_stars_event_min_datetime": "2015-01-09T23:51:16.000Z",
"num_tokens": 68,
"size": 154
} |
-- Concrete definition of variables, context maps, and map operations
module SOAS.Variable {T : Set} where
open import SOAS.Common
open import SOAS.Context
open import SOAS.Sorting
open import SOAS.Families.Core {T}
-- Sorted family of variables, as typed, scoped de Bruijn indices
data ℐ : Familyₛ where
new : {α : T}{Γ : Ctx} → ℐ α (α ∙ Γ)
old : {α β : T}{Γ : Ctx} → ℐ β Γ → ℐ β (α ∙ Γ)
-- Explicitly specify the extra variable type
oldₑ : (α {β} : T)(Γ : Ctx) → ℐ β Γ → ℐ β (α ∙ Γ)
oldₑ α Γ = old {α}{_}{Γ}
open import Relation.Nullary
decEqℐ : ∀ {a b} (x y : ℐ a b) → Dec (x ≡ y)
decEqℐ new new = yes refl
decEqℐ new (old y) = no (λ ())
decEqℐ (old x) new = no (λ ())
decEqℐ (old x) (old y) with decEqℐ x y
... | yes refl = yes refl
... | no npf = no (λ { refl → npf refl })
-- | Context-family maps
-- Generalised transformations between 𝒳-terms in one context and 𝒴-terms in
-- another context. The special case of 𝒳 being the family of variables
-- gives the usual notion of an environment (Allais et al.) or "type preserving
-- map from variables over Γ to stuff over Δ" (McBride 2005), where "stuff" is a
-- sorted family.
-- Context-family map between two sorted families in different contexts.
-- The type is implicitly quantified over.
_~[_➔_]↝_ : Ctx → Familyₛ → Familyₛ → Ctx → Set
Γ ~[ 𝒳 ➔ 𝒴 ]↝ Δ = {τ : T} → 𝒳 τ Γ → 𝒴 τ Δ
-- 𝒳-valued context map, associating variables in context Γ with 𝒳-terms
-- in context Δ.
_~[_]↝_ : Ctx → Familyₛ → Ctx → Set
Γ ~[ 𝒳 ]↝ Δ = Γ ~[ ℐ ➔ 𝒳 ]↝ Δ
infix 10 _~[_]↝_
-- Renaming map, mapping variables to variables
_↝_ : Ctx → Ctx → Set
Γ ↝ Δ = Γ ~[ ℐ ]↝ Δ
infix 4 _↝_
| {
"alphanum_fraction": 0.6406345333,
"avg_line_length": 31.5192307692,
"ext": "agda",
"hexsha": "936d5dfddc54087f18d372c3b0267bed27e20819",
"lang": "Agda",
"max_forks_count": null,
"max_forks_repo_forks_event_max_datetime": null,
"max_forks_repo_forks_event_min_datetime": null,
"max_forks_repo_head_hexsha": "ff1a985a6be9b780d3ba2beff68e902394f0a9d8",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "JoeyEremondi/agda-soas",
"max_forks_repo_path": "SOAS/Variable.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "ff1a985a6be9b780d3ba2beff68e902394f0a9d8",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "JoeyEremondi/agda-soas",
"max_issues_repo_path": "SOAS/Variable.agda",
"max_line_length": 80,
"max_stars_count": null,
"max_stars_repo_head_hexsha": "ff1a985a6be9b780d3ba2beff68e902394f0a9d8",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "JoeyEremondi/agda-soas",
"max_stars_repo_path": "SOAS/Variable.agda",
"max_stars_repo_stars_event_max_datetime": null,
"max_stars_repo_stars_event_min_datetime": null,
"num_tokens": 614,
"size": 1639
} |
{-# OPTIONS --prop --without-K --rewriting #-}
open import Calf.CostMonoid
-- Upper bound on the cost of a computation.
module Calf.Types.Bounded (costMonoid : CostMonoid) where
open CostMonoid costMonoid
open import Calf.Prelude
open import Calf.Metalanguage
open import Calf.PhaseDistinction
open import Calf.Types.Eq
open import Calf.Step costMonoid
open import Calf.Types.Bool
open import Calf.Types.Sum
open import Relation.Binary.PropositionalEquality as Eq
record IsBounded (A : tp pos) (e : cmp (F A)) (c : cmp cost) : □ where
constructor ⇓_withCost_[_,_]
field
result : val A
c' : ℂ
h-bounded : ◯ (c' ≤ c)
h-≡ : cmp (F (eq (U (F A)) e (step (F A) c' (ret result))))
IsBounded⁻ : (A : tp pos) → cmp (F A) → cmp cost → tp neg
IsBounded⁻ A e p = meta (IsBounded A e p)
bound/relax : ∀ {A e p p'} → ◯ (p ≤ p') → IsBounded A e p → IsBounded A e p'
bound/relax h (⇓ result withCost c' [ h-bounded , h-≡ ]) = ⇓ result withCost c' [ (λ u → ≤-trans (h-bounded u) (h u)) , h-≡ ]
bound/circ : ∀ {A e} d {c} →
IsBounded A e c →
IsBounded A e (step (meta ℂ) d c)
bound/circ d {c} (⇓ a withCost c' [ h-bounded , h-≡ ]) =
⇓ a withCost c' [ (λ u → subst (c' ≤_) (sym (step/ext cost c d u)) (h-bounded u)) , h-≡ ]
bound/ret : {A : tp pos} {a : val A} → IsBounded A (ret {A} a) zero
bound/ret {a = a} = ⇓ a withCost zero [ (λ u → ≤-refl) , ret (eq/intro refl) ]
bound/step : ∀ {A e} (d c : ℂ) →
IsBounded A e c →
IsBounded A (step (F A) d e) (d + c)
bound/step d c (⇓ a withCost c' [ h-bounded , h-≡ ]) with eq/ref h-≡
... | refl = ⇓ a withCost d + c' [ (λ u → +-monoʳ-≤ d (h-bounded u)) , ret (eq/intro refl) ]
bound/bind : ∀ {A B : tp pos} {e : cmp (F A)} {f : val A → cmp (F B)}
(c : ℂ) (d : val A → ℂ) →
IsBounded A e c →
((a : val A) → IsBounded B (f a) (d a)) →
IsBounded B (bind {A} (F B) e f)
(bind {A} cost e (λ a → c + d a))
bound/bind {f = f} c d (⇓ a withCost c' [ h-bounded₁ , h-≡₁ ]) h with eq/ref h-≡₁
... | refl with h a
... | ⇓ b withCost d' [ h-bounded₂ , h-≡₂ ] with f a | eq/ref h-≡₂
... | _ | refl = bound/circ c' (⇓ b withCost c' + d' [ (λ u → +-mono-≤ (h-bounded₁ u) (h-bounded₂ u)) , ret (eq/intro refl) ])
bound/bind/const : ∀ {A B : tp pos} {e : cmp (F A)} {f : val A → cmp (F B)}
(c d : ℂ) →
IsBounded A e c →
((a : val A) → IsBounded B (f a) d) →
IsBounded B (bind {A} (F B) e f) (c + d)
bound/bind/const c d (⇓ a withCost c' [ h-bounded , h-≡ ]) h with eq/ref h-≡
... | refl = bound/circ' c' (bound/bind c (λ _ → d) (⇓ a withCost c' [ h-bounded , h-≡ ]) h)
where
bound/circ' : ∀ {A e} d {c} →
IsBounded A e (step (meta ℂ) d c) →
IsBounded A e c
bound/circ' d {c} (⇓ a withCost c' [ h-bounded , h-≡ ]) =
⇓ a withCost c' [ (λ u → subst (c' ≤_) (step/ext cost c d u) (h-bounded u)) , h-≡ ]
bound/bool : ∀ {A : tp pos} {e0 e1} {p : val bool → cmp cost} →
(b : val bool) →
IsBounded A e0 (p false) →
IsBounded A e1 (p true ) →
IsBounded A (if b then e1 else e0) (p b)
bound/bool false h0 h1 = h0
bound/bool true h0 h1 = h1
bound/sum/case/const/const : ∀ A B (C : val (sum A B) → tp pos) →
(s : val (sum A B)) →
(e0 : (a : val A) → cmp (F (C (inj₁ a)))) →
(e1 : (b : val B) → cmp (F (C (inj₂ b)))) →
(p : ℂ) →
((a : val A) → IsBounded (C (inj₁ a)) (e0 a) p) →
((b : val B) → IsBounded (C (inj₂ b)) (e1 b) p) →
IsBounded (C s) (sum/case A B (λ s → F (C s)) s e0 e1) p
bound/sum/case/const/const A B C s e0 e1 p h1 h2 = sum/case A B
(λ s → meta (IsBounded (C s) (sum/case A B (λ s₁ → F (C s₁)) s e0 e1) p)) s h1 h2
| {
"alphanum_fraction": 0.5509974712,
"avg_line_length": 37.0729166667,
"ext": "agda",
"hexsha": "7a510226a5e26061579a74b344ecc3710a1032bb",
"lang": "Agda",
"max_forks_count": 2,
"max_forks_repo_forks_event_max_datetime": "2022-01-29T08:12:01.000Z",
"max_forks_repo_forks_event_min_datetime": "2021-10-06T10:28:24.000Z",
"max_forks_repo_head_hexsha": "e51606f9ca18d8b4cf9a63c2d6caa2efc5516146",
"max_forks_repo_licenses": [
"Apache-2.0"
],
"max_forks_repo_name": "jonsterling/agda-calf",
"max_forks_repo_path": "src/Calf/Types/Bounded.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "e51606f9ca18d8b4cf9a63c2d6caa2efc5516146",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"Apache-2.0"
],
"max_issues_repo_name": "jonsterling/agda-calf",
"max_issues_repo_path": "src/Calf/Types/Bounded.agda",
"max_line_length": 126,
"max_stars_count": 29,
"max_stars_repo_head_hexsha": "e51606f9ca18d8b4cf9a63c2d6caa2efc5516146",
"max_stars_repo_licenses": [
"Apache-2.0"
],
"max_stars_repo_name": "jonsterling/agda-calf",
"max_stars_repo_path": "src/Calf/Types/Bounded.agda",
"max_stars_repo_stars_event_max_datetime": "2022-03-22T20:35:11.000Z",
"max_stars_repo_stars_event_min_datetime": "2021-07-14T03:18:28.000Z",
"num_tokens": 1544,
"size": 3559
} |
module Allto where
f : Set → Set
f = {!!}
g : Set → Set
g x = f {!!}
| {
"alphanum_fraction": 0.4788732394,
"avg_line_length": 8.875,
"ext": "agda",
"hexsha": "d411b0181ea47742a92085316fdf75d1b218101e",
"lang": "Agda",
"max_forks_count": 371,
"max_forks_repo_forks_event_max_datetime": "2022-03-30T19:00:30.000Z",
"max_forks_repo_forks_event_min_datetime": "2015-01-03T14:04:08.000Z",
"max_forks_repo_head_hexsha": "231d6ad8e77b67ff8c4b1cb35a6c31ccd988c3e9",
"max_forks_repo_licenses": [
"BSD-3-Clause"
],
"max_forks_repo_name": "Agda-zh/agda",
"max_forks_repo_path": "test/interaction/Allto.agda",
"max_issues_count": 4066,
"max_issues_repo_head_hexsha": "ed8ac6f4062ea8a20fa0f62d5db82d4e68278338",
"max_issues_repo_issues_event_max_datetime": "2022-03-31T21:14:49.000Z",
"max_issues_repo_issues_event_min_datetime": "2015-01-10T11:24:51.000Z",
"max_issues_repo_licenses": [
"BSD-3-Clause"
],
"max_issues_repo_name": "shlevy/agda",
"max_issues_repo_path": "test/interaction/Allto.agda",
"max_line_length": 18,
"max_stars_count": 1989,
"max_stars_repo_head_hexsha": "ed8ac6f4062ea8a20fa0f62d5db82d4e68278338",
"max_stars_repo_licenses": [
"BSD-3-Clause"
],
"max_stars_repo_name": "shlevy/agda",
"max_stars_repo_path": "test/interaction/Allto.agda",
"max_stars_repo_stars_event_max_datetime": "2022-03-30T18:20:48.000Z",
"max_stars_repo_stars_event_min_datetime": "2015-01-09T23:51:16.000Z",
"num_tokens": 27,
"size": 71
} |
module FFI.Data.Maybe where
{-# FOREIGN GHC import qualified Data.Maybe #-}
data Maybe (A : Set) : Set where
nothing : Maybe A
just : A → Maybe A
{-# COMPILE GHC Maybe = data Data.Maybe.Maybe (Data.Maybe.Nothing|Data.Maybe.Just) #-}
| {
"alphanum_fraction": 0.6861924686,
"avg_line_length": 26.5555555556,
"ext": "agda",
"hexsha": "b16fa810f61a413b703136e32278a0d8db6cd01b",
"lang": "Agda",
"max_forks_count": null,
"max_forks_repo_forks_event_max_datetime": null,
"max_forks_repo_forks_event_min_datetime": null,
"max_forks_repo_head_hexsha": "5187e64f88953f34785ffe58acd0610ee5041f5f",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "FreakingBarbarians/luau",
"max_forks_repo_path": "prototyping/FFI/Data/Maybe.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "5187e64f88953f34785ffe58acd0610ee5041f5f",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "FreakingBarbarians/luau",
"max_issues_repo_path": "prototyping/FFI/Data/Maybe.agda",
"max_line_length": 86,
"max_stars_count": 1,
"max_stars_repo_head_hexsha": "cd18adc20ecb805b8eeb770a9e5ef8e0cd123734",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "Tr4shh/Roblox-Luau",
"max_stars_repo_path": "prototyping/FFI/Data/Maybe.agda",
"max_stars_repo_stars_event_max_datetime": "2022-02-11T21:30:17.000Z",
"max_stars_repo_stars_event_min_datetime": "2022-02-11T21:30:17.000Z",
"num_tokens": 62,
"size": 239
} |
-- Andreas, 2017-07-28, issue #1077
-- Agda's reconstruction of the top-level module can be confusing
-- in case the user puts some illegal declarations before the
-- top level module in error.
foo = Set
module Issue1077 where
bar = Set
-- WAS: accepted, creating modules Issue1077 and Issue1077.Issue1077
-- with Issue1077.foo and Issue1077.Issue1077.bar
-- NOW: Error
-- Illegal declarations before top-level module
| {
"alphanum_fraction": 0.7552941176,
"avg_line_length": 25,
"ext": "agda",
"hexsha": "19618846125ce393b585847bc61f77257573b920",
"lang": "Agda",
"max_forks_count": 371,
"max_forks_repo_forks_event_max_datetime": "2022-03-30T19:00:30.000Z",
"max_forks_repo_forks_event_min_datetime": "2015-01-03T14:04:08.000Z",
"max_forks_repo_head_hexsha": "7f58030124fa99dfbf8db376659416f3ad8384de",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "cruhland/agda",
"max_forks_repo_path": "test/Fail/Issue1077.agda",
"max_issues_count": 4066,
"max_issues_repo_head_hexsha": "7f58030124fa99dfbf8db376659416f3ad8384de",
"max_issues_repo_issues_event_max_datetime": "2022-03-31T21:14:49.000Z",
"max_issues_repo_issues_event_min_datetime": "2015-01-10T11:24:51.000Z",
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "cruhland/agda",
"max_issues_repo_path": "test/Fail/Issue1077.agda",
"max_line_length": 68,
"max_stars_count": 1989,
"max_stars_repo_head_hexsha": "7f58030124fa99dfbf8db376659416f3ad8384de",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "cruhland/agda",
"max_stars_repo_path": "test/Fail/Issue1077.agda",
"max_stars_repo_stars_event_max_datetime": "2022-03-30T18:20:48.000Z",
"max_stars_repo_stars_event_min_datetime": "2015-01-09T23:51:16.000Z",
"num_tokens": 112,
"size": 425
} |
{-# OPTIONS --safe #-}
module Cubical.Algebra.Matrix where
open import Cubical.Foundations.Prelude
open import Cubical.Foundations.Function
open import Cubical.Foundations.Equiv
open import Cubical.Foundations.Structure
open import Cubical.Foundations.Isomorphism
open import Cubical.Foundations.Univalence
open import Cubical.Foundations.HLevels
open import Cubical.Foundations.Transport
open import Cubical.Functions.FunExtEquiv
import Cubical.Data.Empty as ⊥
open import Cubical.Data.Bool
open import Cubical.Data.Nat hiding (_+_ ; _·_; +-comm ; +-assoc; ·-assoc)
open import Cubical.Data.Vec
open import Cubical.Data.Sigma.Base
open import Cubical.Data.FinData
open import Cubical.Relation.Nullary
open import Cubical.Algebra.Group
open import Cubical.Algebra.AbGroup
open import Cubical.Algebra.Monoid
open import Cubical.Algebra.Ring
open import Cubical.Algebra.Ring.BigOps
open Iso
private
variable
ℓ : Level
A : Type ℓ
-- Equivalence between Vec matrix and Fin function matrix
FinMatrix : (A : Type ℓ) (m n : ℕ) → Type ℓ
FinMatrix A m n = FinVec (FinVec A n) m
VecMatrix : (A : Type ℓ) (m n : ℕ) → Type ℓ
VecMatrix A m n = Vec (Vec A n) m
FinMatrix→VecMatrix : {m n : ℕ} → FinMatrix A m n → VecMatrix A m n
FinMatrix→VecMatrix M = FinVec→Vec (λ fm → FinVec→Vec (M fm))
VecMatrix→FinMatrix : {m n : ℕ} → VecMatrix A m n → FinMatrix A m n
VecMatrix→FinMatrix M fn fm = lookup fm (lookup fn M)
FinMatrix→VecMatrix→FinMatrix : {m n : ℕ} (M : FinMatrix A m n)
→ VecMatrix→FinMatrix (FinMatrix→VecMatrix M) ≡ M
FinMatrix→VecMatrix→FinMatrix {m = zero} M = funExt (⊥.rec ∘ ¬Fin0)
FinMatrix→VecMatrix→FinMatrix {n = zero} M = funExt₂ (λ _ → ⊥.rec ∘ ¬Fin0)
FinMatrix→VecMatrix→FinMatrix {m = suc m} {n = suc n} M = funExt₂ goal
where
goal : (fm : Fin (suc m)) (fn : Fin (suc n))
→ VecMatrix→FinMatrix (_ ∷ FinMatrix→VecMatrix (M ∘ suc)) fm fn ≡ M fm fn
goal zero zero = refl
goal zero (suc fn) i = FinVec→Vec→FinVec (M zero ∘ suc) i fn
goal (suc fm) fn i = FinMatrix→VecMatrix→FinMatrix (M ∘ suc) i fm fn
VecMatrix→FinMatrix→VecMatrix : {m n : ℕ} (M : VecMatrix A m n)
→ FinMatrix→VecMatrix (VecMatrix→FinMatrix M) ≡ M
VecMatrix→FinMatrix→VecMatrix {m = zero} [] = refl
VecMatrix→FinMatrix→VecMatrix {m = suc m} (M ∷ MS) i =
Vec→FinVec→Vec M i ∷ VecMatrix→FinMatrix→VecMatrix MS i
FinMatrixIsoVecMatrix : (A : Type ℓ) (m n : ℕ) → Iso (FinMatrix A m n) (VecMatrix A m n)
fun (FinMatrixIsoVecMatrix A m n) = FinMatrix→VecMatrix
inv (FinMatrixIsoVecMatrix A m n) = VecMatrix→FinMatrix
rightInv (FinMatrixIsoVecMatrix A m n) = VecMatrix→FinMatrix→VecMatrix
leftInv (FinMatrixIsoVecMatrix A m n) = FinMatrix→VecMatrix→FinMatrix
FinMatrix≃VecMatrix : {m n : ℕ} → FinMatrix A m n ≃ VecMatrix A m n
FinMatrix≃VecMatrix {_} {A} {m} {n} = isoToEquiv (FinMatrixIsoVecMatrix A m n)
FinMatrix≡VecMatrix : (A : Type ℓ) (m n : ℕ) → FinMatrix A m n ≡ VecMatrix A m n
FinMatrix≡VecMatrix _ _ _ = ua FinMatrix≃VecMatrix
-- Define abelian group structure on matrices
module FinMatrixAbGroup (G' : AbGroup ℓ) where
open AbGroupStr (snd G') renaming ( is-set to isSetG )
private G = ⟨ G' ⟩
zeroFinMatrix : ∀ {m n} → FinMatrix G m n
zeroFinMatrix _ _ = 0g
negFinMatrix : ∀ {m n} → FinMatrix G m n → FinMatrix G m n
negFinMatrix M i j = - M i j
addFinMatrix : ∀ {m n} → FinMatrix G m n → FinMatrix G m n → FinMatrix G m n
addFinMatrix M N i j = M i j + N i j
isSetFinMatrix : ∀ {m n} → isSet (FinMatrix G m n)
isSetFinMatrix = isSetΠ2 λ _ _ → isSetG
addFinMatrixAssoc : ∀ {m n} → (M N K : FinMatrix G m n)
→ addFinMatrix M (addFinMatrix N K) ≡ addFinMatrix (addFinMatrix M N) K
addFinMatrixAssoc M N K i j k = assoc (M j k) (N j k) (K j k) i
addFinMatrix0r : ∀ {m n} → (M : FinMatrix G m n)
→ addFinMatrix M zeroFinMatrix ≡ M
addFinMatrix0r M i j k = rid (M j k) i
addFinMatrix0l : ∀ {m n} → (M : FinMatrix G m n)
→ addFinMatrix zeroFinMatrix M ≡ M
addFinMatrix0l M i j k = lid (M j k) i
addFinMatrixNegMatrixr : ∀ {m n} → (M : FinMatrix G m n)
→ addFinMatrix M (negFinMatrix M) ≡ zeroFinMatrix
addFinMatrixNegMatrixr M i j k = invr (M j k) i
addFinMatrixNegMatrixl : ∀ {m n} → (M : FinMatrix G m n)
→ addFinMatrix (negFinMatrix M) M ≡ zeroFinMatrix
addFinMatrixNegMatrixl M i j k = invl (M j k) i
addFinMatrixComm : ∀ {m n} → (M N : FinMatrix G m n)
→ addFinMatrix M N ≡ addFinMatrix N M
addFinMatrixComm M N i k l = comm (M k l) (N k l) i
FinMatrixAbGroup : (m n : ℕ) → AbGroup ℓ
FinMatrixAbGroup m n =
makeAbGroup {G = FinMatrix G m n} zeroFinMatrix addFinMatrix negFinMatrix
isSetFinMatrix addFinMatrixAssoc addFinMatrix0r
addFinMatrixNegMatrixr addFinMatrixComm
-- Define a abelian group structure on vector matrices and prove that
-- it is equal to FinMatrixAbGroup using the SIP
module _ (G' : AbGroup ℓ) where
open AbGroupStr (snd G')
private G = ⟨ G' ⟩
zeroVecMatrix : ∀ {m n} → VecMatrix G m n
zeroVecMatrix = replicate (replicate 0g)
negVecMatrix : ∀ {m n} → VecMatrix G m n → VecMatrix G m n
negVecMatrix = map (map (λ x → - x))
addVec : ∀ {m} → Vec G m → Vec G m → Vec G m
addVec [] [] = []
addVec (x ∷ xs) (y ∷ ys) = x + y ∷ addVec xs ys
addVecMatrix : ∀ {m n} → VecMatrix G m n → VecMatrix G m n → VecMatrix G m n
addVecMatrix [] [] = []
addVecMatrix (M ∷ MS) (N ∷ NS) = addVec M N ∷ addVecMatrix MS NS
open FinMatrixAbGroup
-- Proof that FinMatrix→VecMatrix is a group homorphism
FinMatrix→VecMatrixHomAdd : (m n : ℕ) (M N : FinMatrix G m n)
→ FinMatrix→VecMatrix (addFinMatrix G' M N) ≡
addVecMatrix (FinMatrix→VecMatrix M) (FinMatrix→VecMatrix N)
FinMatrix→VecMatrixHomAdd zero n M N = refl
FinMatrix→VecMatrixHomAdd (suc m) n M N =
λ i → lem n (M zero) (N zero) i
∷ FinMatrix→VecMatrixHomAdd m n (λ i j → M (suc i) j) (λ i j → N (suc i) j) i
where
lem : (n : ℕ) (V W : FinVec G n)
→ FinVec→Vec (λ j → V j + W j) ≡ addVec (FinVec→Vec V) (FinVec→Vec W)
lem zero V W = refl
lem (suc n) V W = λ i → V zero + W zero ∷ lem n (V ∘ suc) (W ∘ suc) i
-- Combine everything to get an induced abelian group structure of
-- VecMatrix that is equal to the one on FinMatrix
VecMatrixAbGroup : (m n : ℕ) → AbGroup ℓ
VecMatrixAbGroup m n =
InducedAbGroup (FinMatrixAbGroup G' m n) addVecMatrix
FinMatrix≃VecMatrix (FinMatrix→VecMatrixHomAdd m n)
FinMatrixAbGroup≡VecMatrixAbGroup : (m n : ℕ) → FinMatrixAbGroup G' m n ≡ VecMatrixAbGroup m n
FinMatrixAbGroup≡VecMatrixAbGroup m n =
InducedAbGroupPath (FinMatrixAbGroup G' m n) addVecMatrix
FinMatrix≃VecMatrix (FinMatrix→VecMatrixHomAdd m n)
-- Define identity matrix and matrix multiplication for FinMatrix and
-- prove that square matrices form a ring
module _ (R' : Ring ℓ) where
open RingStr (snd R') renaming ( is-set to isSetR )
open RingTheory R'
open KroneckerDelta R'
open Sum R'
open FinMatrixAbGroup (_ , abgroupstr _ _ _ (snd R' .RingStr.+IsAbGroup))
private R = ⟨ R' ⟩
oneFinMatrix : ∀ {n} → FinMatrix R n n
oneFinMatrix i j = δ i j
mulFinMatrix : ∀ {m1 m2 m3} → FinMatrix R m1 m2 → FinMatrix R m2 m3 → FinMatrix R m1 m3
mulFinMatrix M N i k = ∑ λ j → M i j · N j k
∑Exchange : ∀ {m n} → (M : FinMatrix R m n) → ∑ (λ i → ∑ (λ j → M i j)) ≡ ∑ (λ j → ∑ (λ i → M i j))
∑Exchange {m = zero} {n = n} M = sym (∑0r n)
∑Exchange {m = suc m} {n = zero} M = cong (λ x → 0r + x) (∑0r m) ∙ +Rid 0r
∑Exchange {m = suc m} {n = suc n} M =
let a = M zero zero
L = ∑ λ j → M zero (suc j)
C = ∑ λ i → M (suc i) zero
N = ∑ λ i → ∑ λ j → M (suc i) (suc j)
-- N reindexed
N' = ∑ λ j → ∑ λ i → M (suc i) (suc j)
in a + L + ∑ (λ i → ∑ (λ j → M (suc i) j)) ≡⟨ (λ k → a + L + ∑Split (λ i → M (suc i) zero) (λ i → ∑ (λ j → M (suc i) (suc j))) k) ⟩
a + L + (C + N) ≡⟨ (λ k → a + L + (C + ∑Exchange (λ i j → M (suc i) (suc j)) k)) ⟩
a + L + (C + N') ≡⟨ sym (+Assoc _ _ _) ⟩
a + (L + (C + N')) ≡⟨ (λ k → a + +Assoc-comm1 L C N' k) ⟩
a + (C + (L + N')) ≡⟨ +Assoc _ _ _ ⟩
a + C + (L + N') ≡⟨ (λ k → a + C + ∑Split (λ j → M zero (suc j)) (λ j → ∑ (λ i → M (suc i) (suc j))) (~ k)) ⟩
a + C + ∑ (λ j → ∑ (λ i → M i (suc j))) ∎
mulFinMatrixAssoc : ∀ {m n k l} → (M : FinMatrix R m n) → (N : FinMatrix R n k) → (K : FinMatrix R k l)
→ mulFinMatrix M (mulFinMatrix N K) ≡ mulFinMatrix (mulFinMatrix M N) K
mulFinMatrixAssoc M N K = funExt₂ λ i j →
∑ (λ k → M i k · ∑ (λ l → N k l · K l j)) ≡⟨ ∑Ext (λ k → ∑Mulrdist (M i k) (λ l → N k l · K l j)) ⟩
∑ (λ k → ∑ (λ l → M i k · (N k l · K l j))) ≡⟨ ∑Ext (λ k → ∑Ext (λ l → ·Assoc (M i k) (N k l) (K l j))) ⟩
∑ (λ k → ∑ (λ l → M i k · N k l · K l j)) ≡⟨ ∑Exchange (λ k l → M i k · N k l · K l j) ⟩
∑ (λ l → ∑ (λ k → M i k · N k l · K l j)) ≡⟨ ∑Ext (λ l → sym (∑Mulldist (K l j) (λ k → M i k · N k l))) ⟩
∑ (λ l → ∑ (λ k → M i k · N k l) · K l j) ∎
mulFinMatrixr1 : ∀ {m n} → (M : FinMatrix R m n) → mulFinMatrix M oneFinMatrix ≡ M
mulFinMatrixr1 M = funExt₂ λ i j → ∑Mulr1 _ (M i) j
mulFinMatrix1r : ∀ {m n} → (M : FinMatrix R m n) → mulFinMatrix oneFinMatrix M ≡ M
mulFinMatrix1r M = funExt₂ λ i j → ∑Mul1r _ (λ x → M x j) i
mulFinMatrixrDistrAddFinMatrix : ∀ {n} (M N K : FinMatrix R n n)
→ mulFinMatrix M (addFinMatrix N K) ≡ addFinMatrix (mulFinMatrix M N) (mulFinMatrix M K)
mulFinMatrixrDistrAddFinMatrix M N K = funExt₂ λ i j →
∑ (λ k → M i k · (N k j + K k j)) ≡⟨ ∑Ext (λ k → ·Rdist+ (M i k) (N k j) (K k j)) ⟩
∑ (λ k → M i k · N k j + M i k · K k j) ≡⟨ ∑Split (λ k → M i k · N k j) (λ k → M i k · K k j) ⟩
∑ (λ k → M i k · N k j) + ∑ (λ k → M i k · K k j) ∎
mulFinMatrixlDistrAddFinMatrix : ∀ {n} (M N K : FinMatrix R n n)
→ mulFinMatrix (addFinMatrix M N) K ≡ addFinMatrix (mulFinMatrix M K) (mulFinMatrix N K)
mulFinMatrixlDistrAddFinMatrix M N K = funExt₂ λ i j →
∑ (λ k → (M i k + N i k) · K k j) ≡⟨ ∑Ext (λ k → ·Ldist+ (M i k) (N i k) (K k j)) ⟩
∑ (λ k → M i k · K k j + N i k · K k j) ≡⟨ ∑Split (λ k → M i k · K k j) (λ k → N i k · K k j) ⟩
∑ (λ k → M i k · K k j) + ∑ (λ k → N i k · K k j) ∎
FinMatrixRing : (n : ℕ) → Ring ℓ
FinMatrixRing n =
makeRing {R = FinMatrix R n n} zeroFinMatrix oneFinMatrix addFinMatrix
mulFinMatrix negFinMatrix isSetFinMatrix addFinMatrixAssoc
addFinMatrix0r addFinMatrixNegMatrixr addFinMatrixComm
mulFinMatrixAssoc mulFinMatrixr1 mulFinMatrix1r
mulFinMatrixrDistrAddFinMatrix mulFinMatrixlDistrAddFinMatrix
| {
"alphanum_fraction": 0.5956750863,
"avg_line_length": 44.024,
"ext": "agda",
"hexsha": "cef98de17538165ab77fbc3c181e9beba05ea885",
"lang": "Agda",
"max_forks_count": 134,
"max_forks_repo_forks_event_max_datetime": "2022-03-23T16:22:13.000Z",
"max_forks_repo_forks_event_min_datetime": "2018-11-16T06:11:03.000Z",
"max_forks_repo_head_hexsha": "53e159ec2e43d981b8fcb199e9db788e006af237",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "marcinjangrzybowski/cubical",
"max_forks_repo_path": "Cubical/Algebra/Matrix.agda",
"max_issues_count": 584,
"max_issues_repo_head_hexsha": "53e159ec2e43d981b8fcb199e9db788e006af237",
"max_issues_repo_issues_event_max_datetime": "2022-03-30T12:09:17.000Z",
"max_issues_repo_issues_event_min_datetime": "2018-10-15T09:49:02.000Z",
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "marcinjangrzybowski/cubical",
"max_issues_repo_path": "Cubical/Algebra/Matrix.agda",
"max_line_length": 140,
"max_stars_count": 301,
"max_stars_repo_head_hexsha": "53e159ec2e43d981b8fcb199e9db788e006af237",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "marcinjangrzybowski/cubical",
"max_stars_repo_path": "Cubical/Algebra/Matrix.agda",
"max_stars_repo_stars_event_max_datetime": "2022-03-24T02:10:47.000Z",
"max_stars_repo_stars_event_min_datetime": "2018-10-17T18:00:24.000Z",
"num_tokens": 4133,
"size": 11006
} |
open import Common.IO
open import Common.Nat
open import Common.String
open import Common.Unit
private
n : Nat
n = 7
{-# COMPILE OCaml n as val n : Z.t #-}
main : IO Unit
main = do
putStrLn (natToString n)
| {
"alphanum_fraction": 0.6651785714,
"avg_line_length": 14,
"ext": "agda",
"hexsha": "38060e1a5286aa00bd517c0e7fae04d54716211a",
"lang": "Agda",
"max_forks_count": null,
"max_forks_repo_forks_event_max_datetime": null,
"max_forks_repo_forks_event_min_datetime": null,
"max_forks_repo_head_hexsha": "026a8f8473ab91f99c3f6545728e71fa847d2720",
"max_forks_repo_licenses": [
"BSD-3-Clause"
],
"max_forks_repo_name": "xekoukou/agda-ocaml",
"max_forks_repo_path": "test/Compiler/simple/Issue2914.agda",
"max_issues_count": 16,
"max_issues_repo_head_hexsha": "026a8f8473ab91f99c3f6545728e71fa847d2720",
"max_issues_repo_issues_event_max_datetime": "2019-09-08T13:47:04.000Z",
"max_issues_repo_issues_event_min_datetime": "2018-10-08T00:32:04.000Z",
"max_issues_repo_licenses": [
"BSD-3-Clause"
],
"max_issues_repo_name": "xekoukou/agda-ocaml",
"max_issues_repo_path": "test/Compiler/simple/Issue2914.agda",
"max_line_length": 38,
"max_stars_count": 7,
"max_stars_repo_head_hexsha": "026a8f8473ab91f99c3f6545728e71fa847d2720",
"max_stars_repo_licenses": [
"BSD-3-Clause"
],
"max_stars_repo_name": "xekoukou/agda-ocaml",
"max_stars_repo_path": "test/Compiler/simple/Issue2914.agda",
"max_stars_repo_stars_event_max_datetime": "2018-11-06T16:38:43.000Z",
"max_stars_repo_stars_event_min_datetime": "2018-11-05T22:13:36.000Z",
"num_tokens": 64,
"size": 224
} |
-- Minimal implicational logic, PHOAS approach, final encoding
module Pf.ArrMp where
-- Types
infixr 0 _=>_
data Ty : Set where
UNIT : Ty
_=>_ : Ty -> Ty -> Ty
-- Context and truth judgement
Cx : Set1
Cx = Ty -> Set
isTrue : Ty -> Cx -> Set
isTrue a tc = tc a
-- Terms
TmRepr : Set1
TmRepr = Cx -> Ty -> Set
module ArrMp where
record Tm (tr : TmRepr) : Set1 where
infixl 1 _$_
field
var : forall {tc a} -> isTrue a tc -> tr tc a
lam' : forall {tc a b} -> (isTrue a tc -> tr tc b) -> tr tc (a => b)
_$_ : forall {tc a b} -> tr tc (a => b) -> tr tc a -> tr tc b
lam'' : forall {tc a b} -> (tr tc a -> tr tc b) -> tr tc (a => b)
lam'' f = lam' \x -> f (var x)
syntax lam'' (\a -> b) = lam a => b
open Tm {{...}} public
Thm : Ty -> Set1
Thm a = forall {tr tc} {{_ : Tm tr}} -> tr tc a
open ArrMp public
-- Example theorems
aI : forall {a} -> Thm (a => a)
aI =
lam x => x
aK : forall {a b} -> Thm (a => b => a)
aK =
lam x =>
lam _ => x
aS : forall {a b c} -> Thm ((a => b => c) => (a => b) => a => c)
aS =
lam f =>
lam g =>
lam x => f $ x $ (g $ x)
tSKK : forall {a} -> Thm (a => a)
tSKK {a = a} =
aS {b = a => a} $ aK $ aK
| {
"alphanum_fraction": 0.4778761062,
"avg_line_length": 18.552238806,
"ext": "agda",
"hexsha": "33c9fd38a750dc06545e741b5d207b5cddc43280",
"lang": "Agda",
"max_forks_count": null,
"max_forks_repo_forks_event_max_datetime": null,
"max_forks_repo_forks_event_min_datetime": null,
"max_forks_repo_head_hexsha": "2dd761bfa96ccda089888e8defa6814776fa2922",
"max_forks_repo_licenses": [
"X11"
],
"max_forks_repo_name": "mietek/formal-logic",
"max_forks_repo_path": "src/Pf/ArrMp.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "2dd761bfa96ccda089888e8defa6814776fa2922",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"X11"
],
"max_issues_repo_name": "mietek/formal-logic",
"max_issues_repo_path": "src/Pf/ArrMp.agda",
"max_line_length": 75,
"max_stars_count": 26,
"max_stars_repo_head_hexsha": "2dd761bfa96ccda089888e8defa6814776fa2922",
"max_stars_repo_licenses": [
"X11"
],
"max_stars_repo_name": "mietek/formal-logic",
"max_stars_repo_path": "src/Pf/ArrMp.agda",
"max_stars_repo_stars_event_max_datetime": "2021-11-13T12:37:44.000Z",
"max_stars_repo_stars_event_min_datetime": "2015-08-31T09:49:52.000Z",
"num_tokens": 485,
"size": 1243
} |
{-# OPTIONS --prop #-}
postulate
P : Prop
p : P
-- C-c C-n should print `p` as `_`
record Box (X : Prop) : Set where
constructor box
field unbox : X
open Box
test : P → Box P
test = λ x → box x
-- C-c C-n should print `test` as `λ x → box _`
| {
"alphanum_fraction": 0.5725490196,
"avg_line_length": 14.1666666667,
"ext": "agda",
"hexsha": "fe432c4e902046aafee4b5036bd6bb6dbaf9683c",
"lang": "Agda",
"max_forks_count": 371,
"max_forks_repo_forks_event_max_datetime": "2022-03-30T19:00:30.000Z",
"max_forks_repo_forks_event_min_datetime": "2015-01-03T14:04:08.000Z",
"max_forks_repo_head_hexsha": "231d6ad8e77b67ff8c4b1cb35a6c31ccd988c3e9",
"max_forks_repo_licenses": [
"BSD-3-Clause"
],
"max_forks_repo_name": "Agda-zh/agda",
"max_forks_repo_path": "test/interaction/Issue3337.agda",
"max_issues_count": 4066,
"max_issues_repo_head_hexsha": "ed8ac6f4062ea8a20fa0f62d5db82d4e68278338",
"max_issues_repo_issues_event_max_datetime": "2022-03-31T21:14:49.000Z",
"max_issues_repo_issues_event_min_datetime": "2015-01-10T11:24:51.000Z",
"max_issues_repo_licenses": [
"BSD-3-Clause"
],
"max_issues_repo_name": "shlevy/agda",
"max_issues_repo_path": "test/interaction/Issue3337.agda",
"max_line_length": 47,
"max_stars_count": 1989,
"max_stars_repo_head_hexsha": "ed8ac6f4062ea8a20fa0f62d5db82d4e68278338",
"max_stars_repo_licenses": [
"BSD-3-Clause"
],
"max_stars_repo_name": "shlevy/agda",
"max_stars_repo_path": "test/interaction/Issue3337.agda",
"max_stars_repo_stars_event_max_datetime": "2022-03-30T18:20:48.000Z",
"max_stars_repo_stars_event_min_datetime": "2015-01-09T23:51:16.000Z",
"num_tokens": 89,
"size": 255
} |
-- Andreas, 2017-01-21, issue #2424
-- {-# OPTIONS -v tc.cover:40 #-}
-- {-# OPTIONS -v interaction.case:40 #-}
postulate Nat : Set
data List : Set₁ where
_∷_ : (x : Set) (xs : List) → List
test : (As : List) (x : Nat) → Set
test As x = {!As!} -- C-c C-c
-- Expected output:
-- test (x₁ ∷ As) x = {!!}
| {
"alphanum_fraction": 0.536977492,
"avg_line_length": 19.4375,
"ext": "agda",
"hexsha": "8f56a50c9fe40cb6308e12159cf6e0cad08de789",
"lang": "Agda",
"max_forks_count": 371,
"max_forks_repo_forks_event_max_datetime": "2022-03-30T19:00:30.000Z",
"max_forks_repo_forks_event_min_datetime": "2015-01-03T14:04:08.000Z",
"max_forks_repo_head_hexsha": "231d6ad8e77b67ff8c4b1cb35a6c31ccd988c3e9",
"max_forks_repo_licenses": [
"BSD-3-Clause"
],
"max_forks_repo_name": "Agda-zh/agda",
"max_forks_repo_path": "test/interaction/Issue2424.agda",
"max_issues_count": 4066,
"max_issues_repo_head_hexsha": "ed8ac6f4062ea8a20fa0f62d5db82d4e68278338",
"max_issues_repo_issues_event_max_datetime": "2022-03-31T21:14:49.000Z",
"max_issues_repo_issues_event_min_datetime": "2015-01-10T11:24:51.000Z",
"max_issues_repo_licenses": [
"BSD-3-Clause"
],
"max_issues_repo_name": "shlevy/agda",
"max_issues_repo_path": "test/interaction/Issue2424.agda",
"max_line_length": 41,
"max_stars_count": 1989,
"max_stars_repo_head_hexsha": "ed8ac6f4062ea8a20fa0f62d5db82d4e68278338",
"max_stars_repo_licenses": [
"BSD-3-Clause"
],
"max_stars_repo_name": "shlevy/agda",
"max_stars_repo_path": "test/interaction/Issue2424.agda",
"max_stars_repo_stars_event_max_datetime": "2022-03-30T18:20:48.000Z",
"max_stars_repo_stars_event_min_datetime": "2015-01-09T23:51:16.000Z",
"num_tokens": 117,
"size": 311
} |
{- Byzantine Fault Tolerant Consensus Verification in Agda, version 0.9.
Copyright (c) 2021, Oracle and/or its affiliates.
Licensed under the Universal Permissive License v 1.0 as shown at https://opensource.oracle.com/licenses/upl
-}
open import LibraBFT.Base.Types
open import LibraBFT.Concrete.Records
open import LibraBFT.Concrete.System
open import LibraBFT.Concrete.System.Parameters
open import LibraBFT.Impl.Consensus.EpochManager
import LibraBFT.Impl.Consensus.BlockStorage.BlockStore as BlockStore
import LibraBFT.Impl.Consensus.BlockStorage.Properties.BlockStore as BlockStoreProps
import LibraBFT.Impl.Consensus.ConsensusTypes.ExecutedBlock as ExecutedBlock
import LibraBFT.Impl.Consensus.Liveness.RoundState as RoundState
import LibraBFT.Impl.Consensus.Liveness.ProposerElection as ProposerElection
import LibraBFT.Impl.Consensus.PersistentLivenessStorage as PersistentLivenessStorage
import LibraBFT.Impl.Consensus.PersistentLivenessStorage.Properties as PersistentLivenessStorageProps
open import LibraBFT.Impl.Consensus.RoundManager
import LibraBFT.Impl.Consensus.SafetyRules.SafetyRules as SafetyRules
import LibraBFT.Impl.Consensus.SafetyRules.Properties.SafetyRules as SafetyRulesProps
open import LibraBFT.Impl.OBM.Logging.Logging
open import LibraBFT.Impl.Properties.Util
open import LibraBFT.ImplShared.Base.Types
open import LibraBFT.ImplShared.Consensus.Types
open import LibraBFT.ImplShared.Consensus.Types.EpochDep
open import LibraBFT.ImplShared.Interface.Output
open import LibraBFT.ImplShared.Util.Dijkstra.All
open import Optics.All
open import Util.ByteString
open import Util.Hash
open import Util.Lemmas
open import Util.Prelude
open import Yasm.System ℓ-RoundManager ℓ-VSFP ConcSysParms
open OutputProps
open Invariants
open RoundManagerTransProps
-- This module contains properties that are only about the behavior of the handlers, nothing to do
-- with system state
module LibraBFT.Impl.Consensus.RoundManager.Properties where
module executeAndVoteMSpec (vb : ValidBlock) where
b = vbBlock vb
open executeAndVoteM b
open SafetyRulesProps
open import LibraBFT.Impl.Consensus.BlockStorage.Properties.BlockStore
isbQc = (_≡ b ^∙ bQuorumCert)
VoteResultCorrect : (pre post : RoundManager) (lvr≡? : Bool) (r : Either ErrLog Vote) → Set
VoteResultCorrect pre post lvr≡? (Left _) =
VoteNotGenerated pre post lvr≡? ⊎ Voting.VoteGeneratedUnsavedCorrect pre post b
VoteResultCorrect pre post lvr≡? (Right vote) =
Voting.VoteGeneratedCorrect pre post vote b
module _ (pre : RoundManager) where
open QCProps
open Invariants.Reqs b (pre ^∙ lBlockTree)
record Contract (r : Either ErrLog Vote) (post : RoundManager) (outs : List Output) : Set where
constructor mkContract
field
-- General properties / invariants
rmInv : Preserves RoundManagerInv pre post
noEpochChange : NoEpochChange pre post
noMsgOuts : OutputProps.NoMsgs outs
-- Voting
lvr≡? : Bool
voteResultCorrect : NoHC1 → VoteResultCorrect pre post lvr≡? r
-- QCs
qcPost : ∈Post⇒∈PreOr isbQc pre post
contract' :
LBFT-weakestPre (executeAndVoteM b) Contract pre
contract' =
executeAndInsertBlockMSpec.contract vb pre Post₀
(λ where e ._ refl → contractBail [] refl)
contract₁
where
Post₀ : LBFT-Post (Either ErrLog ExecutedBlock)
Post₀ = RWS-weakestPre-∙^∙Post unit (withErrCtx ("" ∷ []))
(RWS-weakestPre-ebindPost unit step₁ Contract)
contractBail : ∀ {e} outs → OutputProps.NoMsgs outs → Contract (Left e) pre outs
contractBail{e} outs noMsgOuts =
mkContract
reflPreservesRoundManagerInv (reflNoEpochChange{pre})
noMsgOuts true (const vrc)
qcPost
where
vrc : VoteResultCorrect pre pre true (Left e)
vrc = inj₁ reflVoteNotGenerated
qcPost : ∈Post⇒∈PreOr isbQc pre pre
qcPost qc = Left
module EAIBM = executeAndInsertBlockMSpec vb
module EAIBE = executeAndInsertBlockESpec (EAIBM.bs pre) vb
module _ (isOk : EAIBE.Ok) (con : EAIBE.ContractOk (proj₁ isOk) (proj₁ (proj₂ isOk))) where
module EAIBECon = EAIBE.ContractOk con
bs' = proj₁ isOk
eb = proj₁ (proj₂ isOk)
pre₁ = pre & rmBlockStore ∙~ bs'
-- State invariants
module _ where
bsP : Preserves BlockStoreInv (rm→BlockStore-EC pre) (rm→BlockStore-EC pre₁)
bsP bsi = EAIBECon.bsInv bsi
srP : Preserves SafetyRulesInv (pre ^∙ lSafetyRules) (pre₁ ^∙ lSafetyRules)
srP = mkPreservesSafetyRulesInv id
invP₁ : Preserves RoundManagerInv pre pre₁
invP₁ = mkPreservesRoundManagerInv id id bsP srP
qcPost-BT : _
qcPost-BT = ∈Post⇒∈PreOrBT-QCs≡ isbQc
(cong (_^∙ bsInner ∙ btHighestCommitCert) EAIBECon.bs≡x)
(cong (_^∙ bsInner ∙ btHighestQuorumCert) EAIBECon.bs≡x)
qcPost₁ : ∈Post⇒∈PreOr isbQc pre pre₁
qcPost₁ = ∈Post⇒∈PreOr-∙-BT-RM isbQc pre pre₁ qcPost-BT
-- For the case any of the checks in `step₁` fails
contractBail₁ : ∀ {e} outs → OutputProps.NoMsgs outs → Contract (Left e) pre₁ outs
contractBail₁ outs noMsgOuts =
mkContract invP₁ refl
noMsgOuts true (const $ inj₁ (mkVoteNotGenerated refl refl))
qcPost₁
contract₁ : Post₀ (Right eb) pre₁ []
proj₁ (contract₁ ._ refl ._ refl ._ refl ._ refl ._ refl) _ = contractBail₁ [] refl
proj₁ (proj₂ (contract₁ ._ refl ._ refl ._ refl ._ refl ._ refl) _) _ = contractBail₁ [] refl
proj₂ (proj₂ (contract₁ ._ refl ._ refl ._ refl ._ refl ._ refl) _) _ = contract₂
where
maybeSignedVoteProposal' = ExecutedBlock.maybeSignedVoteProposal eb
module CASV = constructAndSignVoteMSpec
proposedBlock = CASV.proposedBlock maybeSignedVoteProposal'
Post₂ : LBFT-Post (Either ErrLog Vote)
Post₂ = RWS-weakestPre-ebindPost unit step₃ Contract
contract₂ : RWS-weakestPre (step₂ eb) Contract unit pre₁
contract₂⇒ : RWS-Post-⇒ (CASV.Contract pre₁ proposedBlock) Post₂
contract₂⇒ r pre₃ outs con = contract₂⇒-help r CASVCon.voteResCorrect
where
module CASVCon = CASV.Contract con
CASVouts = outs
invP₂ = transPreservesRoundManagerInv invP₁ CASVCon.rmInv
qcPost₂ : QCProps.∈Post⇒∈PreOr (_≡ b ^∙ bQuorumCert) pre pre₃
qcPost₂ = obm-dangerous-magic' "TODO: waiting on `constructAndSignVoteM` contract"
contract₂⇒-help :
(r : Either ErrLog Vote) (vrc : CASV.VoteResultCorrect pre₁ pre₃ proposedBlock CASVCon.lvr≡? r)
→ RWS-weakestPre-ebindPost unit step₃ Contract r pre₃ outs
contract₂⇒-help (Left _) vrc =
mkContract invP₂ CASVCon.noEpochChange CASVCon.noMsgOuts
CASVCon.lvr≡? (const ∘ Left $ (transVoteNotGenerated (mkVoteNotGenerated refl refl) vrc))
qcPost₂
contract₂⇒-help (Right vote) vrc ._ refl = contract₃
where
open RoundManagerInv
open BlockStoreInv
open BlockTreeInv
contract₃ : RWS-weakestPre (step₃ vote) (RWS-Post++ Contract CASVouts) unit pre₃
contract₃ =
PersistentLivenessStorageProps.saveVoteMSpec.contract vote
Post₃ pre₃
contractBail₃ contractOk₃
where
Post₃ : LBFT-Post (Either ErrLog Unit)
Post₃ = RWS-weakestPre-ebindPost unit (const $ ok vote) (RWS-Post++ Contract CASVouts)
vgc₃ : NoHC1 → Voting.VoteGeneratedCorrect pre pre₃ vote b {- proposedBlock -}
vgc₃ nohc =
Voting.glue-VoteNotGenerated-VoteGeneratedCorrect
(mkVoteNotGenerated refl refl)
(Voting.substVoteGeneratedCorrect proposedBlock b
(EAIBECon.ebBlock≈ nohc)
vrc)
noMsgOutsBail₃ : ∀ outs → NoMsgs outs → NoMsgs (CASVouts ++ outs)
noMsgOutsBail₃ outs noMsgs = ++-NoMsgs CASVouts outs CASVCon.noMsgOuts noMsgs
noMsgOutsOk₃ : ∀ outs → NoMsgs outs → NoMsgs (CASVouts ++ outs ++ [])
noMsgOutsOk₃ outs noMsgs rewrite ++-identityʳ outs = noMsgOutsBail₃ outs noMsgs
contractBail₃ : ∀ outs → NoMsgs outs → NoErrors outs → Post₃ (Left fakeErr) pre₃ outs
contractBail₃ outs noMsgOuts noErrOuts =
mkContract invP₂ CASVCon.noEpochChange (noMsgOutsBail₃ outs noMsgOuts)
CASVCon.lvr≡? ((Right ∘ Voting.mkVoteGeneratedUnsavedCorrect vote) ∘ vgc₃)
qcPost₂
contractOk₃ : ∀ outs → NoMsgs outs → NoErrors outs → Post₃ (Right unit) pre₃ outs
contractOk₃ outs noMsgs noErrs unit refl =
mkContract invP₂ CASVCon.noEpochChange (noMsgOutsOk₃ outs noMsgs)
CASVCon.lvr≡? vgc₃ qcPost₂
contract₂ = constructAndSignVoteMSpec.contract maybeSignedVoteProposal' pre₁ Post₂ contract₂⇒
contract
: ∀ Post
→ RWS-Post-⇒ Contract Post
→ LBFT-weakestPre (executeAndVoteM b) Post pre
contract Post pf =
RWS-⇒ (executeAndVoteM b) unit pre contract' pf
module processProposalMSpec (vproposal : ValidBlock) where
proposal = vbBlock vproposal
open import LibraBFT.Impl.Consensus.BlockStorage.Properties.BlockStore
open import LibraBFT.Impl.Consensus.Liveness.Properties.ProposerElection
open LibraBFT.Impl.Consensus.RoundManager.processProposalM proposal
module _ (pre : RoundManager) where
open Invariants.Reqs (vbBlock vproposal) (pre ^∙ lBlockTree)
record Contract (u : Unit) (post : RoundManager) (outs : List Output) : Set where
constructor mkContract
field
-- General properties / invariants
rmInv : Preserves RoundManagerInv pre post
noEpochChange : NoEpochChange pre post
noProposals : OutputProps.NoProposals outs
-- Voting
voteAttemptCorrect : NoHC1 → Voting.VoteAttemptCorrect pre post outs proposal
-- QCs
outQcs∈RM : QCProps.OutputQc∈RoundManager outs post
qcPost : QCProps.∈Post⇒∈PreOr (_≡ proposal ^∙ bQuorumCert) pre post
contract' : LBFT-weakestPre (processProposalM proposal) Contract pre
contract' ._ refl =
isValidProposalMSpec.contract proposal pre
(RWS-weakestPre-bindPost unit (step₁ (pre ^∙ lBlockStore)) Contract)
(λ where
mAuthor≡nothing ._ refl → (λ _ → contractBail refl) , (λ where ()))
(λ where
notValid ._ refl → (λ _ → contractBail refl) , (λ where ()))
λ where
vp ._ refl →
(λ where ())
, (λ _ →
(λ _ → contractBail refl)
, (λ _ →
(λ _ → contractBail refl)
, (λ _ → contract-step₂)))
where
contractBail : ∀ {outs} → OutputProps.NoMsgs outs → Contract unit pre outs
contractBail{outs} nmo =
mkContract reflPreservesRoundManagerInv (reflNoEpochChange{pre})
noProposals vac outQcs qcPost
where
noProposals : NoProposals outs
noProposals = OutputProps.NoMsgs⇒NoProposals outs nmo
vac : NoHC1 → Voting.VoteAttemptCorrect pre pre outs proposal
vac _ = Voting.voteAttemptBailed outs (OutputProps.NoMsgs⇒NoVotes outs nmo)
outQcs : QCProps.OutputQc∈RoundManager outs pre
outQcs = QCProps.NoMsgs⇒OutputQc∈RoundManager outs pre nmo
qcPost : QCProps.∈Post⇒∈PreOr _ pre pre
qcPost qc = Left
contract-step₂ : RWS-weakestPre (executeAndVoteM proposal >>= step₂) Contract unit pre
contract-step₂ =
executeAndVoteMSpec.contract vproposal pre
(RWS-weakestPre-bindPost unit step₂ Contract) pf-step₂
where
module EAV = executeAndVoteMSpec vproposal
pf-step₂ : RWS-Post-⇒ (EAV.Contract pre) (RWS-weakestPre-bindPost unit step₂ Contract)
pf-step₂ r st outs con = pf r EAVSpec.voteResultCorrect
where
module EAVSpec = executeAndVoteMSpec.Contract con
rmInv₂ = transPreservesRoundManagerInv reflPreservesRoundManagerInv EAVSpec.rmInv
pf : (r : Either ErrLog Vote) (vrc : NoHC1 → EAV.VoteResultCorrect pre st EAVSpec.lvr≡? r)
→ RWS-weakestPre-bindPost unit step₂ Contract r st outs
pf (Left _) vrc ._ refl =
mkContract rmInv₂ EAVSpec.noEpochChange
noProposals
vac
qcOuts EAVSpec.qcPost
where
noMsgs : NoMsgs (outs ++ LogErr _ ∷ [])
noMsgs = ++-NoMsgs outs (LogErr _ ∷ []) EAVSpec.noMsgOuts refl
noProposals : NoProposals (outs ++ LogErr _ ∷ [])
noProposals = NoMsgs⇒NoProposals (outs ++ LogErr _ ∷ []) noMsgs
vac : NoHC1 → Voting.VoteAttemptCorrect pre st (outs ++ LogErr _ ∷ []) proposal
vac nohc =
inj₁ (EAVSpec.lvr≡?
, Voting.mkVoteUnsentCorrect
(NoMsgs⇒NoVotes (outs ++ LogErr _ ∷ []) noMsgs) (vrc nohc))
qcOuts : QCProps.OutputQc∈RoundManager (outs ++ LogErr _ ∷ []) st
qcOuts = QCProps.NoMsgs⇒OutputQc∈RoundManager (outs ++ LogErr _ ∷ []) st noMsgs
pf (Right vote) vrc ._ refl ._ refl ._ refl =
syncInfoMSpec.contract (st & rsVoteSent-rm ?~ vote)
(RWS-weakestPre-bindPost unit (step₃ vote) (RWS-Post++ Contract outs))
contract-step₃
where
stUpdateRS = st & rsVoteSent-rm ?~ vote
module _
(si : SyncInfo)
(si≡ : si ≡ SyncInfo∙new
(st ^∙ lBlockStore ∙ bsHighestQuorumCert)
(st ^∙ lBlockStore ∙ bsHighestCommitCert)
(st ^∙ lBlockStore ∙ bsHighestTimeoutCert))
where
contract-step₃ : RWS-weakestPre (step₃ vote si) (RWS-Post++ Contract outs) unit stUpdateRS
contract-step₃ ._ refl ._ refl ._ refl ._ refl recipient@._ refl =
mkContract rmInv₃
(transNoEpochChange{i = pre}{j = st}{k = stUpdateRS} EAVSpec.noEpochChange refl)
(OutputProps.++-NoProposals outs _ (OutputProps.NoMsgs⇒NoProposals outs EAVSpec.noMsgOuts) refl)
vac
outQcs qcPost
where
vm = VoteMsg∙new vote si
vac : NoHC1 → Voting.VoteAttemptCorrect pre stUpdateRS (outs ++ SendVote vm _ ∷ []) proposal
vac nohc =
inj₂ (Voting.mkVoteSentCorrect vm recipient
(OutputProps.++-NoVotes-OneVote outs _ (OutputProps.NoMsgs⇒NoVotes outs EAVSpec.noMsgOuts) refl)
(Voting.glue-VoteGeneratedCorrect-VoteNotGenerated{s₂ = st}
(vrc nohc) (mkVoteNotGenerated refl refl)))
outQcs : QCProps.OutputQc∈RoundManager (outs ++ SendVote vm _ ∷ []) stUpdateRS
outQcs =
QCProps.++-OutputQc∈RoundManager{stUpdateRS}{outs}
(QCProps.NoMsgs⇒OutputQc∈RoundManager outs stUpdateRS EAVSpec.noMsgOuts)
(outQcSendVote ∷ [])
where
outQcSendVote : ∀ qc nm → qc QC∈NM nm → nm Msg∈Out (SendVote vm _) → qc QCProps.∈RoundManager stUpdateRS
outQcSendVote qc .(V (VoteMsg∙new vote si)) (inSI inV (withVoteSIHighQC qc≡)) inSV rewrite si≡ =
QCProps.inHQC (sym qc≡)
outQcSendVote qc .(V (VoteMsg∙new vote si)) (inSI inV (withVoteSIHighCC qc≡)) inSV =
QCProps.inHCC (just-injective $
begin
just qc ≡⟨ lem₁ ⟩
sixxx ≡⟨ lem₂ (cong is-just (sym lem₁)) ⟩
just (stUpdateRS ^∙ lBlockStore ∙ bsInner ∙ btHighestCommitCert) ∎)
where
open ≡-Reasoning
sixxx = if (st ^∙ lBlockStore ∙ bsHighestQuorumCert) QCBoolEq (st ^∙ lBlockStore ∙ bsHighestCommitCert)
then nothing
else (just $ (st ^∙ lBlockStore ∙ bsHighestCommitCert))
lem₁ : just qc ≡ sixxx
lem₁ = begin
just qc ≡⟨ sym qc≡ ⟩
vm ^∙ vmSyncInfo ∙ sixxxHighestCommitCert ≡⟨ cong (_^∙ sixxxHighestCommitCert) si≡ ⟩
sixxx ∎
lem₂ : is-just sixxx ≡ true
→ sixxx ≡ just (stUpdateRS ^∙ lBlockStore ∙ bsInner ∙ btHighestCommitCert)
lem₂ isj
with (st ^∙ lBlockStore ∙ bsHighestQuorumCert) QCBoolEq (st ^∙ lBlockStore ∙ bsHighestCommitCert)
... | false = refl
... | true = absurd false ≡ true case isj of λ ()
qcPost : QCProps.∈Post⇒∈PreOr (_≡ proposal ^∙ bQuorumCert) pre stUpdateRS
qcPost qc qc∈stUpdateRS = EAVSpec.qcPost qc (qc∈st qc∈stUpdateRS)
where
qc∈st : qc QCProps.∈RoundManager stUpdateRS → qc QCProps.∈RoundManager st
qc∈st (QCProps.inHQC qc≡) = QCProps.inHQC qc≡
qc∈st (QCProps.inHCC qc≡) = QCProps.inHCC qc≡
-- state invariants
module _ where
bsP : Preserves BlockStoreInv (rm→BlockStore-EC st) (rm→BlockStore-EC stUpdateRS)
bsP = id
srP : Preserves SafetyRulesInv (st ^∙ lSafetyRules) (stUpdateRS ^∙ lSafetyRules)
srP = mkPreservesSafetyRulesInv id
rmInv₃ : Preserves RoundManagerInv pre stUpdateRS
rmInv₃ = transPreservesRoundManagerInv rmInv₂
(mkPreservesRoundManagerInv id id bsP srP)
contract : ∀ Post → RWS-Post-⇒ Contract Post → LBFT-weakestPre (processProposalM proposal) Post pre
contract Post pf = LBFT-⇒ (processProposalM proposal) pre contract' pf
module syncUpMSpec
(now : Instant) (syncInfo : SyncInfo) (author : Author) (_helpRemote : Bool) where
open syncUpM now syncInfo author _helpRemote
open import LibraBFT.Impl.Consensus.ConsensusTypes.Properties.SyncInfo
open import LibraBFT.Impl.Consensus.BlockStorage.Properties.SyncManager
module _ (pre : RoundManager) where
record Contract (r : Either ErrLog Unit) (post : RoundManager) (outs : List Output) : Set where
constructor mkContract
field
-- General invariants / properties
rmInv : Preserves RoundManagerInv pre post
dnmBtIdToBlk : post ≡L pre at (lBlockTree ∙ btIdToBlock)
noEpochChange : NoEpochChange pre post
noVoteOuts : OutputProps.NoVotes outs
-- Voting
noVote : VoteNotGenerated pre post true
-- QCs
noOutQcs : QCProps.¬OutputQc outs
qcPost : QCProps.∈Post⇒∈PreOr (_QC∈SyncInfo syncInfo) pre post
contract' : LBFT-weakestPre (syncUpM now syncInfo author _helpRemote) Contract pre
contract' =
BlockStoreProps.syncInfoMSpec.contract pre
(RWS-weakestPre-bindPost unit step₁ Contract)
contract₁
where
localSyncInfo = BlockStoreProps.syncInfoMSpec.syncInfo pre
contract₁ : RWS-weakestPre-bindPost unit step₁ Contract (BlockStoreProps.syncInfoMSpec.syncInfo pre) pre []
proj₂ (contract₁ localSyncInfo lsi≡) hnc≡false =
mkContract reflPreservesRoundManagerInv refl (reflNoEpochChange{pre}) refl
(reflVoteNotGenerated{pre})
[] qcPost
where
outQcs : QCProps.OutputQc∈RoundManager [] pre
outQcs = QCProps.NoMsgs⇒OutputQc∈RoundManager [] pre refl
qcPost : QCProps.∈Post⇒∈PreOr _ pre pre
qcPost qc = Left
proj₁ (contract₁ localSyncInfo lsi≡) hcn≡true vv@._ refl =
verifyMSpec.contract syncInfo vv pre Post₁
contract₃
where
Post₁ : LBFT-Post (Either ErrLog Unit)
Post₁ = (RWS-weakestPre-∙^∙Post unit (withErrCtx (here' []))
(RWS-weakestPre-ebindPost unit (λ _ → step₃ localSyncInfo vv) Contract))
contract₃ : RWS-Post-⇒ (verifyMSpec.Contract syncInfo vv pre) Post₁
contract₃ r st outs con ._ refl
with VSpec.noStateChange
where module VSpec = verifyMSpec.Contract con
contract₃ (Left x) st outs con ._ refl
| refl
= mkContract VSpec.rmInv (cong (_^∙ lBlockTree ∙ btIdToBlock) VSpec.noStateChange) (reflNoEpochChange{st})
(++-NoVotes outs [] (NoMsgs⇒NoVotes outs VSpec.noMsgOuts) refl)
(reflVoteNotGenerated{st})
noOutQcs qcPost
where
module VSpec = verifyMSpec.Contract con
noOutQcs : QCProps.¬OutputQc (outs ++ [])
noOutQcs = QCProps.++-¬OutputQc (QCProps.NoMsgs⇒¬OutputQc outs VSpec.noMsgOuts) []
qcPost : QCProps.∈Post⇒∈PreOr _ st st
qcPost qc = Left
contract₃ (Right y) st₃ outs₃ con₃ ._ refl
| refl = λ where
unit refl →
addCertsMSpec.contract syncInfo retriever st₃
Post₃ contract₄
where
Post₃ : LBFT-Post (Either ErrLog Unit)
Post₃ = (RWS-weakestPre-∙^∙Post unit (withErrCtx (here' []))
(RWS-weakestPre-ebindPost unit (λ _ → step₄ localSyncInfo vv)
(RWS-Post++ Contract (outs₃ ++ []))))
retriever = BlockRetriever∙new now author
contract₄ : RWS-Post-⇒ (addCertsMSpec.Contract syncInfo retriever st₃) Post₃
contract₄ (Left _) st₄ outs₄ con₄ ._ refl =
mkContract AC.rmInv AC.dnmBtIdToBlk AC.noEpochChange noVotes₄ AC.noVote noOutQcs AC.qcPost
where
module AC = addCertsMSpec.Contract con₄
module VSpec = verifyMSpec.Contract con₃
noVotes₄ : NoVotes $ (outs₃ ++ []) ++ outs₄ ++ []
noVotes₄ =
++-NoVotes (outs₃ ++ []) (outs₄ ++ [])
(++-NoVotes outs₃ [] (NoMsgs⇒NoVotes outs₃ VSpec.noMsgOuts) refl)
(++-NoVotes outs₄ [] AC.noVoteOuts refl)
noOutQcs : QCProps.¬OutputQc ((outs₃ ++ []) ++ outs₄ ++ [])
noOutQcs =
QCProps.++-¬OutputQc
(QCProps.++-¬OutputQc
(QCProps.NoMsgs⇒¬OutputQc outs₃ VSpec.noMsgOuts)
(QCProps.NoMsgs⇒¬OutputQc [] refl))
(QCProps.++-¬OutputQc
AC.noOutQc (QCProps.NoMsgs⇒¬OutputQc [] refl))
contract₄ (Right _) st₄ outs₄ con₄ ._ refl =
obm-dangerous-magic' "TODO: waiting on contract for `processCertificatesM`"
contract
: ∀ Post → RWS-Post-⇒ Contract Post
→ LBFT-weakestPre (syncUpM now syncInfo author _helpRemote) Post pre
contract Post pf =
LBFT-⇒ (syncUpM now syncInfo author _helpRemote) pre
contract' pf
module ensureRoundAndSyncUpMSpec
(now : Instant) (messageRound : Round) (syncInfo : SyncInfo)
(author : Author) (helpRemote : Bool) where
open ensureRoundAndSyncUpM now messageRound syncInfo author helpRemote
module _ (pre : RoundManager) where
record Contract (r : Either ErrLog Bool) (post : RoundManager) (outs : List Output) : Set where
constructor mkContract
field
-- General invariants / properties
rmInv : Preserves RoundManagerInv pre post
dnmBtIdToBlk : post ≡L pre at (lBlockTree ∙ btIdToBlock)
noEpochChange : NoEpochChange pre post
noVoteOuts : OutputProps.NoVotes outs
-- Voting
noVote : VoteNotGenerated pre post true
-- Signatures
noOutQcs : QCProps.¬OutputQc outs
qcPost : QCProps.∈Post⇒∈PreOr (_QC∈SyncInfo syncInfo) pre post
contract'
: LBFT-weakestPre (ensureRoundAndSyncUpM now messageRound syncInfo author helpRemote) Contract pre
proj₁ (contract' ._ refl) _ =
mkContract id refl refl refl vng outqcs qcPost
where
vng : VoteNotGenerated pre pre true
vng = mkVoteNotGenerated refl refl
outqcs : QCProps.¬OutputQc []
outqcs = []
qcPost : QCProps.∈Post⇒∈PreOr _ pre pre
qcPost qc = Left
proj₂ (contract' ._ refl) mrnd≥crnd = contract-step₁
where
contract-step₁ : LBFT-weakestPre step₁ Contract pre
contract-step₁ = syncUpMSpec.contract now syncInfo author helpRemote pre Post contract-step₁'
where
Post = RWS-weakestPre-ebindPost unit (const step₂) Contract
contract-step₁' : _
contract-step₁' (Left _ ) st outs con =
mkContract SU.rmInv SU.dnmBtIdToBlk SU.noEpochChange SU.noVoteOuts SU.noVote SU.noOutQcs SU.qcPost
where
module SU = syncUpMSpec.Contract con
contract-step₁' (Right unit) st outs con = contract-step₂
where
module SU = syncUpMSpec.Contract con
noVoteOuts' : NoVotes (outs ++ [])
noVoteOuts' = ++-NoVotes outs [] SU.noVoteOuts refl
noOutQcs : QCProps.¬OutputQc (outs ++ [])
noOutQcs =
QCProps.++-¬OutputQc SU.noOutQcs []
contract-step₂ : Post (Right unit) st outs
proj₁ (contract-step₂ ._ refl ._ refl) _ =
mkContract SU.rmInv SU.dnmBtIdToBlk SU.noEpochChange noVoteOuts' SU.noVote
noOutQcs SU.qcPost
proj₂ (contract-step₂ ._ refl ._ refl) _ =
mkContract SU.rmInv SU.dnmBtIdToBlk SU.noEpochChange noVoteOuts' SU.noVote
noOutQcs SU.qcPost
contract : ∀ Post → RWS-Post-⇒ Contract Post → LBFT-weakestPre (ensureRoundAndSyncUpM now messageRound syncInfo author helpRemote) Post pre
contract Post pf =
LBFT-⇒ (ensureRoundAndSyncUpM now messageRound syncInfo author helpRemote) pre contract' pf
module processProposalMsgMSpec
(now : Instant) (pm : ProposalMsg) (vproposal : BlockId-correct (pm ^∙ pmProposal)) where
proposal = pm ^∙ pmProposal
open processProposalMsgM now pm
module _ (pre : RoundManager) where
open Invariants.Reqs proposal (pre ^∙ lBlockTree)
record Contract (_ : Unit) (post : RoundManager) (outs : List Output) : Set where
constructor mkContract
field
-- General invariants / properties
rmInv : Preserves RoundManagerInv pre post
noEpochChange : NoEpochChange pre post
-- Voting
voteAttemptCorrect : NoHC1 → Voting.VoteAttemptCorrect pre post outs proposal
-- QCs
outQcs∈RM : QCProps.OutputQc∈RoundManager outs post
qcPost : QCProps.∈Post⇒∈PreOr (_QC∈NM (P pm)) pre post
contract' : LBFT-weakestPre (processProposalMsgM now pm) Contract pre
contract' rewrite processProposalMsgM≡ = contract
where
contractBail : ∀ outs → OutputProps.NoMsgs outs → Contract unit pre outs
contractBail outs nmo =
mkContract reflPreservesRoundManagerInv (reflNoEpochChange{pre}) vac outqcs qcPost
where
vac : NoHC1 → Voting.VoteAttemptCorrect pre pre outs proposal
vac _ = Voting.voteAttemptBailed outs (OutputProps.NoMsgs⇒NoVotes outs nmo)
outqcs : QCProps.OutputQc∈RoundManager outs pre
outqcs = QCProps.NoMsgs⇒OutputQc∈RoundManager outs pre nmo
qcPost : QCProps.∈Post⇒∈PreOr _ pre pre
qcPost qc = Left
contract : LBFT-weakestPre step₀ Contract pre
proj₁ contract ≡nothing = contractBail _ refl
proj₂ contract = contract-step₁
where
-- These arguments come from the second proof obligation of RWS-weakestPre for RWS-maybe
module _ (pAuthor : Author) (pAuthor≡ : pm ^∙ pmProposer ≡ just pAuthor) where
pf-step₂ : RWS-Post-⇒ _ (RWS-weakestPre-bindPost unit step₂ Contract)
contract-step₁ : LBFT-weakestPre (step₁ pAuthor) Contract pre
contract-step₁ =
ensureRoundAndSyncUpMSpec.contract now (pm ^∙ pmProposal ∙ bRound) (pm ^∙ pmSyncInfo) pAuthor true pre
(RWS-weakestPre-bindPost unit step₂ Contract)
pf-step₂
pf-step₂ r st outs con = pf-step₂' r
where
module ERASU = ensureRoundAndSyncUpMSpec.Contract con
contractBailAfterSync : ∀ outs' → OutputProps.NoMsgs outs' → RWS-Post++ Contract outs unit st outs'
contractBailAfterSync outs' noMsgs' =
mkContract ERASU.rmInv ERASU.noEpochChange vac outqcs qcPost
where
vac : NoHC1 → Voting.VoteAttemptCorrect pre st (outs ++ outs') proposal
vac _ = Left (true , (Voting.mkVoteUnsentCorrect
(OutputProps.++-NoVotes outs _ ERASU.noVoteOuts (OutputProps.NoMsgs⇒NoVotes outs' noMsgs'))
(Left ERASU.noVote)))
outqcs : QCProps.OutputQc∈RoundManager (outs ++ outs') st
outqcs =
QCProps.¬OutputQc⇒OutputQc∈RoundManager (outs ++ outs') st
(QCProps.++-¬OutputQc ERASU.noOutQcs
(QCProps.NoMsgs⇒¬OutputQc outs' noMsgs'))
qcPost : QCProps.∈Post⇒∈PreOr (_QC∈NM (P pm)) pre st
qcPost qc qc∈st
with ERASU.qcPost qc qc∈st
... | Left qc∈pre = Left qc∈pre
... | Right qc∈si = Right (inSI inP qc∈si)
pf-step₂' : (r : Either ErrLog Bool) → RWS-weakestPre-bindPost unit step₂ Contract r st outs
pf-step₂' (Left e) ._ refl =
contractBailAfterSync _ refl
pf-step₂' (Right false) ._ refl ._ refl =
contractBailAfterSync _ refl
pf-step₂' (Right true) ._ refl =
processProposalMSpec.contract (proposal , vproposal)
st
(RWS-Post++ Contract outs)
pf-step₃
where
pf-step₃ : RWS-Post-⇒
(processProposalMSpec.Contract (proposal , vproposal) _)
(RWS-Post++ Contract outs)
pf-step₃ unit st' outs' con =
mkContract
(transPreservesRoundManagerInv ERASU.rmInv (PP.rmInv con))
(transNoEpochChange{i = pre}{j = st}{k = st'} ERASU.noEpochChange (PP.noEpochChange con))
vac outqcs qcPost
where
module PP = processProposalMSpec.Contract
vac : NoHC1 → Voting.VoteAttemptCorrect pre st' (outs ++ outs') proposal
vac nohc rewrite sym ERASU.dnmBtIdToBlk =
Voting.glue-VoteNotGenerated-VoteAttemptCorrect{outs₁ = outs}
ERASU.noVote ERASU.noVoteOuts (PP.voteAttemptCorrect con nohc)
outqcs : QCProps.OutputQc∈RoundManager (outs ++ outs') st'
outqcs =
QCProps.++-OutputQc∈RoundManager {rm = st'}
(QCProps.¬OutputQc⇒OutputQc∈RoundManager outs st' ERASU.noOutQcs)
(PP.outQcs∈RM con)
qcPost : QCProps.∈Post⇒∈PreOr (_QC∈NM (P pm)) pre st'
qcPost qc qc∈st'
with PP.qcPost con qc qc∈st'
...| Right refl = Right inP
...| Left qc∈st
with ERASU.qcPost qc qc∈st
... | Right qc∈si = Right (inSI inP qc∈si)
... | Left qc∈pre = Left qc∈pre
contract : ∀ Post → RWS-Post-⇒ Contract Post → LBFT-weakestPre (processProposalMsgM now pm) Post pre
contract Post pf =
LBFT-⇒ (processProposalMsgM now pm) pre contract' pf
module startSpec
(now : Instant)
(lastVoteSent : Maybe Vote)
where
module _ (pre : RoundManager)
(rmi : RoundManagerInv pre) -- preconditions needed to prove contract
where
open InitProofDefs
open start now lastVoteSent
Contract : LBFT-Post Unit
Contract _ post outs = ∃[ e ] (find' logErrMB outs ≡ just e)
⊎ find' logErrMB outs ≡ nothing × InitContractOk lastVoteSent post outs
syncInfo = SyncInfo∙new (pre ^∙ (lBlockStore ∙ bsHighestQuorumCert))
(pre ^∙ (lBlockStore ∙ bsHighestCommitCert))
(pre ^∙ (lBlockStore ∙ bsHighestTimeoutCert))
postulate
contract-step₁ : LBFT-weakestPre (step₁-abs syncInfo) Contract pre
contract' : LBFT-weakestPre (start-abs now lastVoteSent) Contract pre
-- These are due to the various binds arising from syncInfoM, which is not abstract
-- because it's more trouble than it's worth
contract' rewrite start-abs-≡ =
λ where ._ refl ._ refl ._ refl ._ refl ._ refl ._ refl si refl → contract-step₁
| {
"alphanum_fraction": 0.6143041896,
"avg_line_length": 44.9918809202,
"ext": "agda",
"hexsha": "f0b5914464169077d1f1ace7171de7057a7b34a5",
"lang": "Agda",
"max_forks_count": null,
"max_forks_repo_forks_event_max_datetime": null,
"max_forks_repo_forks_event_min_datetime": null,
"max_forks_repo_head_hexsha": "a4674fc473f2457fd3fe5123af48253cfb2404ef",
"max_forks_repo_licenses": [
"UPL-1.0"
],
"max_forks_repo_name": "LaudateCorpus1/bft-consensus-agda",
"max_forks_repo_path": "src/LibraBFT/Impl/Consensus/RoundManager/Properties.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "a4674fc473f2457fd3fe5123af48253cfb2404ef",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"UPL-1.0"
],
"max_issues_repo_name": "LaudateCorpus1/bft-consensus-agda",
"max_issues_repo_path": "src/LibraBFT/Impl/Consensus/RoundManager/Properties.agda",
"max_line_length": 143,
"max_stars_count": null,
"max_stars_repo_head_hexsha": "a4674fc473f2457fd3fe5123af48253cfb2404ef",
"max_stars_repo_licenses": [
"UPL-1.0"
],
"max_stars_repo_name": "LaudateCorpus1/bft-consensus-agda",
"max_stars_repo_path": "src/LibraBFT/Impl/Consensus/RoundManager/Properties.agda",
"max_stars_repo_stars_event_max_datetime": null,
"max_stars_repo_stars_event_min_datetime": null,
"num_tokens": 9300,
"size": 33249
} |
{-# OPTIONS --universe-polymorphism #-}
open import Categories.Category
module Categories.Object.Coproducts {o ℓ e} (C : Category o ℓ e) where
open Category C
open import Level
import Categories.Object.Initial as Initial
import Categories.Object.BinaryCoproducts as BinaryCoproducts
open Initial C
open BinaryCoproducts C
-- this should really be 'FiniteCoproducts', no?
record Coproducts : Set (o ⊔ ℓ ⊔ e) where
field
initial : Initial
binary : BinaryCoproducts | {
"alphanum_fraction": 0.764091858,
"avg_line_length": 22.8095238095,
"ext": "agda",
"hexsha": "fa84d3c72a3a8a1979025964755fb93c8012c841",
"lang": "Agda",
"max_forks_count": 23,
"max_forks_repo_forks_event_max_datetime": "2021-11-11T13:50:56.000Z",
"max_forks_repo_forks_event_min_datetime": "2015-02-05T13:03:09.000Z",
"max_forks_repo_head_hexsha": "e41aef56324a9f1f8cf3cd30b2db2f73e01066f2",
"max_forks_repo_licenses": [
"BSD-3-Clause"
],
"max_forks_repo_name": "p-pavel/categories",
"max_forks_repo_path": "Categories/Object/Coproducts.agda",
"max_issues_count": 19,
"max_issues_repo_head_hexsha": "e41aef56324a9f1f8cf3cd30b2db2f73e01066f2",
"max_issues_repo_issues_event_max_datetime": "2019-08-09T16:31:40.000Z",
"max_issues_repo_issues_event_min_datetime": "2015-05-23T06:47:10.000Z",
"max_issues_repo_licenses": [
"BSD-3-Clause"
],
"max_issues_repo_name": "p-pavel/categories",
"max_issues_repo_path": "Categories/Object/Coproducts.agda",
"max_line_length": 70,
"max_stars_count": 98,
"max_stars_repo_head_hexsha": "36f4181d751e2ecb54db219911d8c69afe8ba892",
"max_stars_repo_licenses": [
"BSD-3-Clause"
],
"max_stars_repo_name": "copumpkin/categories",
"max_stars_repo_path": "Categories/Object/Coproducts.agda",
"max_stars_repo_stars_event_max_datetime": "2022-03-08T05:20:36.000Z",
"max_stars_repo_stars_event_min_datetime": "2015-04-15T14:57:33.000Z",
"num_tokens": 129,
"size": 479
} |
{-# OPTIONS --without-K --safe #-}
module Categories.Category.Instance.FinCatShapes where
open import Data.Nat using (ℕ)
open import Data.Fin
open import Relation.Binary using (IsEquivalence)
open import Relation.Binary.PropositionalEquality as ≡ using (refl; _≡_; module ≡-Reasoning)
open import Categories.Category
open import Categories.Category.Finite.Fin
open import Categories.Utils.EqReasoning
-- essentially a functor, but we don't need the congruence rule
record FinCatShape⇒ (X Y : FinCatShape) : Set where
private
module X = FinCatShape X
module Y = FinCatShape Y
field
F₀ : Fin X.size → Fin Y.size
F₁ : ∀ {x y} → x X.⇒ y → F₀ x Y.⇒ F₀ y
identity : ∀ {x} → F₁ (X.id {x}) ≡ Y.id
homomorphism : ∀ {x y z} {f : x X.⇒ y} {g : y X.⇒ z} →
F₁ (g X.∘ f) ≡ F₁ g Y.∘ F₁ f
record _≈_ {X Y} (f g : FinCatShape⇒ X Y) : Set where
private
module X = FinCatShape X
module Y = FinCatShape Y
module f = FinCatShape⇒ f
module g = FinCatShape⇒ g
field
F₀≡ : ∀ x → f.F₀ x ≡ g.F₀ x
F₁≡ : ∀ {x y} (w : x X.⇒ y) → ≡.subst₂ Y._⇒_ (F₀≡ x) (F₀≡ y) (f.F₁ w) ≡ g.F₁ w
private
open ≡-Reasoning
id : ∀ {A} → FinCatShape⇒ A A
id {A} = record
{ F₀ = λ x → x
; F₁ = λ x → x
; identity = refl
; homomorphism = refl
}
where open FinCatShape A
comp : ∀ {A B C} → FinCatShape⇒ B C → FinCatShape⇒ A B → FinCatShape⇒ A C
comp {A} {B} {C} f g = record
{ F₀ = λ a → f.F₀ (g.F₀ a)
; F₁ = λ w → f.F₁ (g.F₁ w)
; identity = λ {a} → begin
f.F₁ (g.F₁ A.id) ≡⟨ ≡.cong f.F₁ g.identity ⟩
f.F₁ B.id ≡⟨ f.identity ⟩
C.id ∎
; homomorphism = λ {a b c} {z w} → begin
f.F₁ (g.F₁ (w A.∘ z)) ≡⟨ ≡.cong f.F₁ g.homomorphism ⟩
f.F₁ (g.F₁ w B.∘ g.F₁ z) ≡⟨ f.homomorphism ⟩
f.F₁ (g.F₁ w) C.∘ f.F₁ (g.F₁ z) ∎
}
where module A = FinCatShape A
module B = FinCatShape B
module C = FinCatShape C
module f = FinCatShape⇒ f
module g = FinCatShape⇒ g
assoc : ∀ {A B C D} {f : FinCatShape⇒ A B} {g : FinCatShape⇒ B C} {h : FinCatShape⇒ C D} →
comp (comp h g) f ≈ comp h (comp g f)
assoc {A} {B} {C} {D} {f} {g} {h} = record
{ F₀≡ = λ a → refl
; F₁≡ = λ w → refl
}
where module A = FinCatShape A
module B = FinCatShape B
module C = FinCatShape C
module D = FinCatShape D
module f = FinCatShape⇒ f
module g = FinCatShape⇒ g
module h = FinCatShape⇒ h
identityˡ : ∀ {A B} {f : FinCatShape⇒ A B} → comp id f ≈ f
identityˡ {A} {B} {f} = record
{ F₀≡ = λ x → refl
; F₁≡ = λ w → refl
}
where module A = FinCatShape A
module B = FinCatShape B
module f = FinCatShape⇒ f
identityʳ : ∀ {A B} {f : FinCatShape⇒ A B} → comp f id ≈ f
identityʳ {A} {B} {f} = record
{ F₀≡ = λ x → refl
; F₁≡ = λ w → refl
}
where module A = FinCatShape A
module B = FinCatShape B
module f = FinCatShape⇒ f
equiv : ∀ {A B} → IsEquivalence (_≈_ {A} {B})
equiv {A} {B} = record
{ refl = record
{ F₀≡ = λ x → refl
; F₁≡ = λ w → refl
}
; sym = λ {x y} eq →
let module x = FinCatShape⇒ x
module y = FinCatShape⇒ y
open _≈_ eq
in record
{ F₀≡ = λ z → ≡.sym (F₀≡ z)
; F₁≡ = λ {a b} w → begin
≡.subst₂ B._⇒_ (≡.sym (F₀≡ a)) (≡.sym (F₀≡ b)) (y.F₁ w)
≡˘⟨ ≡.cong (≡.subst₂ B._⇒_ (≡.sym (F₀≡ a)) (≡.sym (F₀≡ b))) (F₁≡ w) ⟩
≡.subst₂ B._⇒_ (≡.sym (F₀≡ a)) (≡.sym (F₀≡ b)) (≡.subst₂ B._⇒_ (F₀≡ a) (F₀≡ b) (x.F₁ w))
≡⟨ subst₂-sym-subst₂ B._⇒_ (F₀≡ a) (F₀≡ b) ⟩
x.F₁ w
∎
}
; trans = λ {x y z} eq eq′ →
let module x = FinCatShape⇒ x
module y = FinCatShape⇒ y
module z = FinCatShape⇒ z
module eq = _≈_ eq
module eq′ = _≈_ eq′
in record
{ F₀≡ = λ a → ≡.trans (eq.F₀≡ a) (eq′.F₀≡ a)
; F₁≡ = λ {a b} w → begin
≡.subst₂ B._⇒_ (≡.trans (eq.F₀≡ a) (eq′.F₀≡ a)) (≡.trans (eq.F₀≡ b) (eq′.F₀≡ b)) (x.F₁ w)
≡˘⟨ subst₂-subst₂ B._⇒_ (eq.F₀≡ a) (eq′.F₀≡ a) (eq.F₀≡ b) (eq′.F₀≡ b) ⟩
≡.subst₂ B._⇒_ (eq′.F₀≡ a) (eq′.F₀≡ b) (≡.subst₂ B._⇒_ (eq.F₀≡ a) (eq.F₀≡ b) (x.F₁ w))
≡⟨ ≡.cong (≡.subst₂ B._⇒_ (eq′.F₀≡ a) (eq′.F₀≡ b)) (eq.F₁≡ w) ⟩
≡.subst₂ B._⇒_ (eq′.F₀≡ a) (eq′.F₀≡ b) (y.F₁ w)
≡⟨ eq′.F₁≡ w ⟩
z.F₁ w
∎
}
}
where module A = FinCatShape A
module B = FinCatShape B
∘-resp-≈ : ∀ {A B C} {f h : FinCatShape⇒ B C} {g i : FinCatShape⇒ A B} →
f ≈ h → g ≈ i → comp f g ≈ comp h i
∘-resp-≈ {A} {B} {C} {f} {h} {g} {i} eq eq′ = record
{ F₀≡ = λ a → ≡.trans (≡.cong f.F₀ (eq′.F₀≡ a)) (eq.F₀≡ (i.F₀ a))
; F₁≡ = λ {x y} w → begin
≡.subst₂ C._⇒_
(≡.trans (≡.cong f.F₀ (eq′.F₀≡ x)) (eq.F₀≡ (i.F₀ x)))
(≡.trans (≡.cong f.F₀ (eq′.F₀≡ y)) (eq.F₀≡ (i.F₀ y)))
(F₁ (comp f g) w)
≡˘⟨ subst₂-subst₂ C._⇒_ (≡.cong f.F₀ (eq′.F₀≡ x)) (eq.F₀≡ (i.F₀ x)) (≡.cong f.F₀ (eq′.F₀≡ y)) (eq.F₀≡ (i.F₀ y)) ⟩
≡.subst₂ C._⇒_ (eq.F₀≡ (i.F₀ x)) (eq.F₀≡ (i.F₀ y))
(≡.subst₂ C._⇒_ (≡.cong f.F₀ (eq′.F₀≡ x)) (≡.cong f.F₀ (eq′.F₀≡ y))
(F₁ (comp f g) w))
≡⟨ ≡.cong (≡.subst₂ C._⇒_ (eq.F₀≡ (i.F₀ x)) (eq.F₀≡ (i.F₀ y))) (subst₂-app C._⇒_ (g.F₁ w) (λ _ _ → f.F₁) (eq′.F₀≡ x) (eq′.F₀≡ y)) ⟩
≡.subst₂ C._⇒_ (eq.F₀≡ (i.F₀ x)) (eq.F₀≡ (i.F₀ y))
(f.F₁ (≡.subst₂ B._⇒_ (eq′.F₀≡ x) (eq′.F₀≡ y) (g.F₁ w)))
≡⟨ ≡.cong (λ j → ≡.subst₂ C._⇒_ (eq.F₀≡ (i.F₀ x)) (eq.F₀≡ (i.F₀ y)) (f.F₁ j)) (eq′.F₁≡ w) ⟩
≡.subst₂ C._⇒_ (eq.F₀≡ (i.F₀ x)) (eq.F₀≡ (i.F₀ y)) (f.F₁ (i.F₁ w))
≡⟨ eq.F₁≡ (i.F₁ w) ⟩
h.F₁ (i.F₁ w)
∎
}
where module A = FinCatShape A
module B = FinCatShape B
module C = FinCatShape C
module f = FinCatShape⇒ f
module g = FinCatShape⇒ g
module h = FinCatShape⇒ h
module i = FinCatShape⇒ i
module eq = _≈_ eq
module eq′ = _≈_ eq′
open FinCatShape⇒
FinCatShapes : Category _ _ _
FinCatShapes = categoryHelper record
{ Obj = FinCatShape
; _⇒_ = FinCatShape⇒
; _≈_ = _≈_
; id = id
; _∘_ = comp
; assoc = λ {A B C D} {f g} {h} → assoc {f = f} {g} {h}
; identityˡ = identityˡ
; identityʳ = identityʳ
; equiv = equiv
; ∘-resp-≈ = ∘-resp-≈
}
| {
"alphanum_fraction": 0.4710221286,
"avg_line_length": 34.5989583333,
"ext": "agda",
"hexsha": "32b1ec6cbb63af5abaefde68ea8fa5baa9ae7df7",
"lang": "Agda",
"max_forks_count": null,
"max_forks_repo_forks_event_max_datetime": null,
"max_forks_repo_forks_event_min_datetime": null,
"max_forks_repo_head_hexsha": "58e5ec015781be5413bdf968f7ec4fdae0ab4b21",
"max_forks_repo_licenses": [
"MIT"
],
"max_forks_repo_name": "MirceaS/agda-categories",
"max_forks_repo_path": "src/Categories/Category/Instance/FinCatShapes.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "58e5ec015781be5413bdf968f7ec4fdae0ab4b21",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"MIT"
],
"max_issues_repo_name": "MirceaS/agda-categories",
"max_issues_repo_path": "src/Categories/Category/Instance/FinCatShapes.agda",
"max_line_length": 139,
"max_stars_count": null,
"max_stars_repo_head_hexsha": "58e5ec015781be5413bdf968f7ec4fdae0ab4b21",
"max_stars_repo_licenses": [
"MIT"
],
"max_stars_repo_name": "MirceaS/agda-categories",
"max_stars_repo_path": "src/Categories/Category/Instance/FinCatShapes.agda",
"max_stars_repo_stars_event_max_datetime": null,
"max_stars_repo_stars_event_min_datetime": null,
"num_tokens": 3076,
"size": 6643
} |
(1 ∷ 4 ∷ []) ∷ (2 ∷ 5 ∷ []) ∷ (3 ∷ 6 ∷ []) ∷ []
| {
"alphanum_fraction": 0.125,
"avg_line_length": 24,
"ext": "agda",
"hexsha": "0e7d98bad3c8f34707e803cb02a2986b6eab6bb1",
"lang": "Agda",
"max_forks_count": 1,
"max_forks_repo_forks_event_max_datetime": "2018-11-09T22:08:40.000Z",
"max_forks_repo_forks_event_min_datetime": "2018-11-09T22:08:40.000Z",
"max_forks_repo_head_hexsha": "9ad63ea473a958506c041077f1d810c0c7c8c18d",
"max_forks_repo_licenses": [
"Info-ZIP"
],
"max_forks_repo_name": "seanwallawalla-forks/RosettaCodeData",
"max_forks_repo_path": "Task/Matrix-transposition/Agda/matrix-transposition-2.agda",
"max_issues_count": null,
"max_issues_repo_head_hexsha": "9ad63ea473a958506c041077f1d810c0c7c8c18d",
"max_issues_repo_issues_event_max_datetime": null,
"max_issues_repo_issues_event_min_datetime": null,
"max_issues_repo_licenses": [
"Info-ZIP"
],
"max_issues_repo_name": "seanwallawalla-forks/RosettaCodeData",
"max_issues_repo_path": "Task/Matrix-transposition/Agda/matrix-transposition-2.agda",
"max_line_length": 47,
"max_stars_count": 1,
"max_stars_repo_head_hexsha": "9ad63ea473a958506c041077f1d810c0c7c8c18d",
"max_stars_repo_licenses": [
"Info-ZIP"
],
"max_stars_repo_name": "LaudateCorpus1/RosettaCodeData",
"max_stars_repo_path": "Task/Matrix-transposition/Agda/matrix-transposition-2.agda",
"max_stars_repo_stars_event_max_datetime": "2018-11-09T22:08:38.000Z",
"max_stars_repo_stars_event_min_datetime": "2018-11-09T22:08:38.000Z",
"num_tokens": 34,
"size": 48
} |
{-# OPTIONS --without-K #-}
module sets.finite.core where
open import sum
open import function.isomorphism
open import sets.nat
open import sets.fin
IsOfSize : ∀ {i} → Set i → ℕ → Set i
IsOfSize A n = A ≅ Fin n
IsFinite : ∀ {i} → Set i → Set i
IsFinite A = Σ ℕ (IsOfSize A)
mk-is-finite : ∀ {i n}{A : Set i}
→ (A ≅ Fin n)
→ IsFinite A
mk-is-finite {n = n} enum = n , enum
fin-is-finite : ∀ {n} → IsFinite (Fin n)
fin-is-finite {n} = mk-is-finite refl≅
⊎-of-size : ∀ {i j n m}{A : Set i}{B : Set j}
→ IsOfSize A n
→ IsOfSize B m
→ IsOfSize (A ⊎ B) (n + m)
⊎-of-size isoA isoB = ⊎-ap-iso isoA isoB ·≅ fin-sum
⊎-finite : ∀ {i j}{A : Set i}{B : Set j}
→ IsFinite A → IsFinite B
→ IsFinite (A ⊎ B)
⊎-finite (_ , fA) (_ , fB) = mk-is-finite (⊎-of-size fA fB)
×-of-size : ∀ {i j n m}{A : Set i}{B : Set j}
→ IsOfSize A n
→ IsOfSize B m
→ IsOfSize (A × B) (n * m)
×-of-size isoA isoB = ×-ap-iso isoA isoB ·≅ fin-prod
×-finite : ∀ {i j}{A : Set i}{B : Set j}
→ IsFinite A → IsFinite B
→ IsFinite (A × B)
×-finite (_ , fA) (_ , fB) = mk-is-finite (×-of-size fA fB)
| {
"alphanum_fraction": 0.518549747,
"avg_line_length": 26.9545454545,
"ext": "agda",
"hexsha": "c00fd625b851bc62a1fe0cd83d8365cd1fdeb95a",
"lang": "Agda",
"max_forks_count": 4,
"max_forks_repo_forks_event_max_datetime": "2019-05-04T19:31:00.000Z",
"max_forks_repo_forks_event_min_datetime": "2015-02-02T12:17:00.000Z",
"max_forks_repo_head_hexsha": "bbbc3bfb2f80ad08c8e608cccfa14b83ea3d258c",
"max_forks_repo_licenses": [
"BSD-3-Clause"
],
"max_forks_repo_name": "pcapriotti/agda-base",
"max_forks_repo_path": "src/sets/finite/core.agda",
"max_issues_count": 4,
"max_issues_repo_head_hexsha": "bbbc3bfb2f80ad08c8e608cccfa14b83ea3d258c",
"max_issues_repo_issues_event_max_datetime": "2016-10-26T11:57:26.000Z",
"max_issues_repo_issues_event_min_datetime": "2015-02-02T14:32:16.000Z",
"max_issues_repo_licenses": [
"BSD-3-Clause"
],
"max_issues_repo_name": "pcapriotti/agda-base",
"max_issues_repo_path": "src/sets/finite/core.agda",
"max_line_length": 59,
"max_stars_count": 20,
"max_stars_repo_head_hexsha": "bbbc3bfb2f80ad08c8e608cccfa14b83ea3d258c",
"max_stars_repo_licenses": [
"BSD-3-Clause"
],
"max_stars_repo_name": "pcapriotti/agda-base",
"max_stars_repo_path": "src/sets/finite/core.agda",
"max_stars_repo_stars_event_max_datetime": "2022-02-01T11:25:54.000Z",
"max_stars_repo_stars_event_min_datetime": "2015-06-12T12:20:17.000Z",
"num_tokens": 459,
"size": 1186
} |
Subsets and Splits
No community queries yet
The top public SQL queries from the community will appear here once available.